Theory Definitions_Main
section‹Main definitions of the development\label{sec:main-definitions}›
theory Definitions_Main
imports
Absolute_Versions
begin
text‹This theory gathers the main definitions of the
\<^session>‹Transitive_Models› session and the present one.
It might be considered as the bare minimum reading requisite to
trust that our development indeed formalizes the theory of
forcing. This should be mathematically clear since this is the
only known method for obtaining proper extensions of ctms while
preserving the ordinals.
The main theorem of this session and all of its relevant definitions
appear in Section~\ref{sec:def-main-forcing}. The reader trusting
all the libraries on which our development is based, might jump
directly to Section~\ref{sec:relative-arith}, which treats relative
cardinal arithmetic as implemented in
\<^session>‹Transitive_Models›. But in case one wants to dive deeper, the
following sections treat some basic concepts of the ZF logic
(Section~\ref{sec:def-main-ZF}) and in the
ZF-Constructible library (Section~\ref{sec:def-main-relative})
on which our definitions are built.
›
declare [[show_question_marks=false]]
subsection‹ZF\label{sec:def-main-ZF}›
text‹For the basic logic ZF we restrict ourselves to just a few
concepts.›
thm bij_def[unfolded inj_def surj_def]
text‹@{thm [display] bij_def[unfolded inj_def surj_def]}›
thm eqpoll_def
text‹@{thm [display] eqpoll_def}›
thm Transset_def
text‹@{thm [display] Transset_def}›
thm Ord_def
text‹@{thm [display] Ord_def}›
thm lt_def le_iff
text‹@{thm [display] lt_def le_iff}›
text‹With the concepts of empty set and successor in place,›
lemma empty_def': "∀x. x ∉ 0" by simp
lemma succ_def': "succ(i) = i ∪ {i}" by blast
text‹we can define the set of natural numbers \<^term>‹ω›. In the
sources, it is defined as a fixpoint, but here we just write
its characterization as the first limit ordinal.›
thm Limit_nat[unfolded Limit_def] nat_le_Limit[unfolded Limit_def]
text‹@{thm [display] Limit_nat[unfolded Limit_def]
nat_le_Limit[unfolded Limit_def]}›
text‹Then, addition and predecessor on \<^term>‹ω› are inductively
characterized as follows:›
thm add_0_right add_succ_right pred_0 pred_succ_eq
text‹@{thm [display] add_succ_right add_0_right pred_0 pred_succ_eq}›
text‹Lists on a set \<^term>‹A› can be characterized by being
recursively generated from the empty list \<^term>‹[]› and the
operation \<^term>‹Cons› that adds a new element to the left end;
the induction theorem for them shows that the characterization is
``complete''.›
thm Nil Cons list.induct
text‹@{thm [display] Nil Cons list.induct }›
text‹Length, concatenation, and \<^term>‹n›th element of lists are
recursively characterized as follows.›
thm length.simps app.simps nth_0 nth_Cons
text‹@{thm [display] length.simps app.simps nth_0 nth_Cons}›
text‹We have the usual Haskell-like notation for iterated applications
of \<^term>‹Cons›:›
lemma Cons_app: "[a,b,c] = Cons(a,Cons(b,Cons(c,[])))" ..
text‹Relative quantifiers restrict the range of the bound variable to a
class \<^term>‹M› of type \<^typ>‹i⇒o›; that is, a truth-valued function with
set arguments.›
lemma "∀x[M]. P(x) ≡ ∀x. M(x) ⟶ P(x)"
"∃x[M]. P(x) ≡ ∃x. M(x) ∧ P(x)"
unfolding rall_def rex_def .
text‹Finally, a set can be viewed (``cast'') as a class using the
following function of type \<^typ>‹i⇒(i⇒o)›.›
thm setclass_iff
text‹@{thm [display] setclass_iff}›
subsection‹Relative concepts\label{sec:def-main-relative}›
text‹A list of relative concepts (mostly from the ZF-Constructible
library) follows next.›
thm big_union_def
text‹@{thm [display] big_union_def}›
thm upair_def
text‹@{thm [display] upair_def}›
thm pair_def
text‹@{thm [display] pair_def}›
thm successor_def[unfolded is_cons_def union_def]
text‹@{thm [display] successor_def[unfolded is_cons_def union_def]}›
thm empty_def
text‹@{thm [display] empty_def}›
thm transitive_set_def[unfolded subset_def]
text‹@{thm [display] transitive_set_def[unfolded subset_def]}›
thm ordinal_def
text‹@{thm [display] ordinal_def}›
thm image_def
text‹@{thm [display] image_def}›
thm fun_apply_def
text‹@{thm [display] fun_apply_def}›
thm is_function_def
text‹@{thm [display] is_function_def}›
thm is_relation_def
text‹@{thm [display] is_relation_def}›
thm is_domain_def
text‹@{thm [display] is_domain_def}›
thm typed_function_def
text‹@{thm [display] typed_function_def}›
thm is_function_space_def[unfolded is_funspace_def]
function_space_rel_def surjection_def
text‹@{thm [display] is_function_space_def[unfolded is_funspace_def]
function_space_rel_def surjection_def}›
text‹Relative version of the $\ZFC$ axioms›
thm extensionality_def
text‹@{thm [display] extensionality_def}›
thm foundation_ax_def
text‹@{thm [display] foundation_ax_def}›
thm upair_ax_def
text‹@{thm [display] upair_ax_def}›
thm Union_ax_def
text‹@{thm [display] Union_ax_def}›
thm power_ax_def[unfolded powerset_def subset_def]
text‹@{thm [display] power_ax_def[unfolded powerset_def subset_def]}›
thm infinity_ax_def
text‹@{thm [display] infinity_ax_def}›
thm choice_ax_def
text‹@{thm [display] choice_ax_def}›
thm separation_def
text‹@{thm [display] separation_def}›
thm univalent_def
text‹@{thm [display] univalent_def}›
thm strong_replacement_def
text‹@{thm [display] strong_replacement_def}›
text‹Internalized formulas›
text‹``Codes'' for formulas (as sets) are constructed from natural
numbers using \<^term>‹Member›, \<^term>‹Equal›, \<^term>‹Nand›,
and \<^term>‹Forall›.›
thm Member Equal Nand Forall formula.induct
text‹@{thm [display] Member Equal Nand Forall formula.induct}›
text‹Definitions for the other connectives and the internal existential
quantifier are also provided. For instance, negation:›
thm Neg_def
text‹@{thm [display] Neg_def}›
thm arity.simps
text‹@{thm [display] arity.simps}›
text‹We have the satisfaction relation between $\in$-models and
first order formulas (given a ``environment'' list representing
the assignment of free variables),›
thm mem_iff_sats equal_iff_sats sats_Nand_iff sats_Forall_iff
text‹@{thm [display] mem_iff_sats equal_iff_sats sats_Nand_iff sats_Forall_iff}›
text‹as well as the satisfaction of an arbitrary set of sentences.›
thm satT_def
text‹@{thm [display] satT_def}›
text‹The internalized (viz. as elements of the set \<^term>‹formula›)
version of the axioms follow next.›
thm ZF_union_iff_sats ZF_power_iff_sats ZF_pairing_iff_sats
ZF_foundation_iff_sats ZF_extensionality_iff_sats
ZF_infinity_iff_sats sats_ZF_separation_fm_iff
sats_ZF_replacement_fm_iff ZF_choice_iff_sats
text‹@{thm [display] ZF_union_iff_sats ZF_power_iff_sats
ZF_pairing_iff_sats
ZF_foundation_iff_sats ZF_extensionality_iff_sats
ZF_infinity_iff_sats sats_ZF_separation_fm_iff
sats_ZF_replacement_fm_iff ZF_choice_iff_sats}›
text‹Above, we use the following:›
thm replacement_assm_def
text‹@{thm [display] replacement_assm_def}›
text‹Finally, the axiom sets are defined as follows.›
thm ZF_fin_def ZF_schemes_def Zermelo_fms_def ZC_def ZF_def ZFC_def
text‹@{thm [display] ZF_fin_def ZF_schemes_def Zermelo_fms_def ZC_def ZF_def
ZFC_def}›
subsection‹Relativization of infinitary arithmetic\label{sec:relative-arith}›
text‹In order to state the defining property of the relative
equipotence relation, we work under the assumptions of the
locale \<^term>‹M_cardinals›. They comprise a finite set
of instances of Separation and Replacement to prove
closure properties of the transitive class \<^term>‹M›.›
lemma (in M_cardinals) eqpoll_def':
assumes "M(A)" "M(B)" shows "A ≈⇗M⇖ B ⟷ (∃f[M]. f ∈ bij(A,B))"
using assms unfolding eqpoll_rel_def by auto
text‹Below, $\mu$ denotes the minimum operator on the ordinals.›
lemma cardinalities_defs:
fixes M::"i⇒o"
shows
"|A|⇗M⇖ ≡ μ i. M(i) ∧ i ≈⇗M⇖ A"
"Card⇗M⇖(α) ≡ α = |α|⇗M⇖"
"κ⇗↑ν,M⇖ ≡ |ν →⇗M⇖ κ|⇗M⇖"
"(κ⇧+)⇗M⇖ ≡ μ x. M(x) ∧ Card⇗M⇖(x) ∧ κ < x"
unfolding cardinal_rel_def cexp_rel_def
csucc_rel_def Card_rel_def .
context M_aleph
begin
text‹Analogous to the previous Lemma @{thm [source] eqpoll_def'}, we are now under
the assumptions of the locale \<^term>‹M_aleph›. The axiom instances
included are sufficient to state and prove the defining
properties of the relativized \<^term>‹Aleph› function
(in particular, the required ability to perform transfinite recursions).›
thm Aleph_rel_zero Aleph_rel_succ Aleph_rel_limit
text‹@{thm [display] Aleph_rel_zero Aleph_rel_succ Aleph_rel_limit}›
end
lemma ContHyp_rel_def':
fixes N::"i⇒o"
shows
"CH⇗N⇖ ≡ ℵ⇘1⇙⇗N⇖ = 2⇗↑ℵ⇘0⇙⇗N⇖,N⇖"
unfolding ContHyp_rel_def .
text‹Under appropriate hypotheses (this time, from the locale \<^term>‹M_ZF_library›),
\<^term>‹CH⇗M⇖› is equivalent to its fully relational version \<^term>‹is_ContHyp›.
As a sanity check, we see that if the transitive class is indeed \<^term>‹𝒱›,
we recover the original $\CH$.›
thm M_ZF_library.is_ContHyp_iff is_ContHyp_iff_CH[unfolded ContHyp_def]
text‹@{thm [display] M_ZF_library.is_ContHyp_iff
is_ContHyp_iff_CH[unfolded ContHyp_def]}›
text‹In turn, the fully relational version evaluated on a nonempty
transitive \<^term>‹A› is equivalent to the satisfaction of the
first-order formula \<^term>‹⋅CH⋅›.›
thm is_ContHyp_iff_sats
text‹@{thm [display] is_ContHyp_iff_sats}›
subsection‹Forcing \label{sec:def-main-forcing}›
text‹Our first milestone was to obtain a proper extension using forcing.
Its original proof didn't required the previous developments involving
the relativization of material on cardinal arithmetic. Now it is
derived from a stronger result, namely @{thm [source] extensions_of_ctms}
below.›
thm extensions_of_ctms_ZF
text‹@{thm [display] extensions_of_ctms_ZF}›
text‹We can finally state our main results, namely, the existence of models
for $\ZFC + \CH$ and $\ZFC + \neg\CH$ under the assumption of a ctm of $\ZFC$.›
thm ctm_ZFC_imp_ctm_not_CH
text‹@{thm [display] ctm_ZFC_imp_ctm_not_CH}›
thm ctm_ZFC_imp_ctm_CH
text‹@{thm [display] ctm_ZFC_imp_ctm_CH}›
text‹These results can be strengthened by enumerating six finite sets of
replacement instances which are sufficient to develop forcing and for
the construction of the aforementioned models: \<^term>‹instances1_fms›
through \<^term>‹instances3_fms›, \<^term>‹instances_ground_fms›, and
\<^term>‹instances_ground_notCH_fms›,
which are then collected into the $31$-element set \<^term>‹overhead_notCH›.
For example, we have:›
thm instances1_fms_def
text‹@{thm [display] instances1_fms_def}›
thm overhead_def overhead_notCH_def
text‹@{thm [display] overhead_def overhead_notCH_def overhead_CH_def}›
text‹One further instance is needed to force $\CH$, with a total count
of $32$ instances:›
thm overhead_CH_def
text‹@{thm [display] overhead_CH_def}›
thm extensions_of_ctms
text‹@{thm [display] extensions_of_ctms}›
thm ctm_of_not_CH
text‹@{thm [display] ctm_of_not_CH}›
thm ctm_of_CH
text‹@{thm [display] ctm_of_CH}›
text‹In the above three statements, the function \<^term>‹ground_repl_fm›
takes an element \<^term>‹φ› of \<^term>‹formula› and returns the
replacement instance in the ground model that produces the
\<^term>‹φ›-replacement instance in the generic extension. The next
result is stated in the context \<^locale>‹G_generic1›, which assumes
the existence of a generic filter.›
context G_generic1
begin
thm sats_ground_repl_fm_imp_sats_ZF_replacement_fm
text‹@{thm [display] sats_ground_repl_fm_imp_sats_ZF_replacement_fm}›
end
end