| author | haftmann | 
| Fri, 16 Mar 2007 21:32:08 +0100 | |
| changeset 22452 | 8a86fd2a1bf0 | 
| parent 21404 | eb85850d3eb7 | 
| child 23755 | 1c4672d130b1 | 
| permissions | -rw-r--r-- | 
| 14706 | 1 | (* Title : HOL/Library/Zorn.thy | 
| 13652 | 2 | ID : $Id$ | 
| 3 | Author : Jacques D. Fleuriot | |
| 14706 | 4 | Description : Zorn's Lemma -- see Larry Paulson's Zorn.thy in ZF | 
| 5 | *) | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 6 | |
| 14706 | 7 | header {* Zorn's Lemma *}
 | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 8 | |
| 15131 | 9 | theory Zorn | 
| 15140 | 10 | imports Main | 
| 15131 | 11 | begin | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 12 | |
| 14706 | 13 | text{*
 | 
| 14 | The lemma and section numbers refer to an unpublished article | |
| 15 |   \cite{Abrial-Laffitte}.
 | |
| 16 | *} | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 17 | |
| 19736 | 18 | definition | 
| 21404 
eb85850d3eb7
more robust syntax for definition/abbreviation/notation;
 wenzelm parents: 
19736diff
changeset | 19 | chain :: "'a set set => 'a set set set" where | 
| 19736 | 20 |   "chain S  = {F. F \<subseteq> S & (\<forall>x \<in> F. \<forall>y \<in> F. x \<subseteq> y | y \<subseteq> x)}"
 | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 21 | |
| 21404 
eb85850d3eb7
more robust syntax for definition/abbreviation/notation;
 wenzelm parents: 
19736diff
changeset | 22 | definition | 
| 
eb85850d3eb7
more robust syntax for definition/abbreviation/notation;
 wenzelm parents: 
19736diff
changeset | 23 | super :: "['a set set,'a set set] => 'a set set set" where | 
| 19736 | 24 |   "super S c = {d. d \<in> chain S & c \<subset> d}"
 | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 25 | |
| 21404 
eb85850d3eb7
more robust syntax for definition/abbreviation/notation;
 wenzelm parents: 
19736diff
changeset | 26 | definition | 
| 
eb85850d3eb7
more robust syntax for definition/abbreviation/notation;
 wenzelm parents: 
19736diff
changeset | 27 | maxchain :: "'a set set => 'a set set set" where | 
| 19736 | 28 |   "maxchain S = {c. c \<in> chain S & super S c = {}}"
 | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 29 | |
| 21404 
eb85850d3eb7
more robust syntax for definition/abbreviation/notation;
 wenzelm parents: 
19736diff
changeset | 30 | definition | 
| 
eb85850d3eb7
more robust syntax for definition/abbreviation/notation;
 wenzelm parents: 
19736diff
changeset | 31 | succ :: "['a set set,'a set set] => 'a set set" where | 
| 19736 | 32 | "succ S c = | 
| 33 | (if c \<notin> chain S | c \<in> maxchain S | |
| 34 | then c else SOME c'. c' \<in> super S c)" | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 35 | |
| 14706 | 36 | consts | 
| 37 | TFin :: "'a set set => 'a set set set" | |
| 38 | inductive "TFin S" | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 39 | intros | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 40 | succI: "x \<in> TFin S ==> succ S x \<in> TFin S" | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 41 | Pow_UnionI: "Y \<in> Pow(TFin S) ==> Union(Y) \<in> TFin S" | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 42 | monos Pow_mono | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 43 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 44 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 45 | subsection{*Mathematical Preamble*}
 | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 46 | |
| 17200 | 47 | lemma Union_lemma0: | 
| 18143 | 48 | "(\<forall>x \<in> C. x \<subseteq> A | B \<subseteq> x) ==> Union(C) \<subseteq> A | B \<subseteq> Union(C)" | 
| 17200 | 49 | by blast | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 50 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 51 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 52 | text{*This is theorem @{text increasingD2} of ZF/Zorn.thy*}
 | 
| 17200 | 53 | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 54 | lemma Abrial_axiom1: "x \<subseteq> succ S x" | 
| 17200 | 55 | apply (unfold succ_def) | 
| 56 | apply (rule split_if [THEN iffD2]) | |
| 57 | apply (auto simp add: super_def maxchain_def psubset_def) | |
| 18585 | 58 | apply (rule contrapos_np, assumption) | 
| 17200 | 59 | apply (rule someI2, blast+) | 
| 60 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 61 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 62 | lemmas TFin_UnionI = TFin.Pow_UnionI [OF PowI] | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 63 | |
| 14706 | 64 | lemma TFin_induct: | 
| 65 | "[| n \<in> TFin S; | |
| 66 | !!x. [| x \<in> TFin S; P(x) |] ==> P(succ S x); | |
| 67 | !!Y. [| Y \<subseteq> TFin S; Ball Y P |] ==> P(Union Y) |] | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 68 | ==> P(n)" | 
| 19736 | 69 | apply (induct set: TFin) | 
| 17200 | 70 | apply blast+ | 
| 71 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 72 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 73 | lemma succ_trans: "x \<subseteq> y ==> x \<subseteq> succ S y" | 
| 17200 | 74 | apply (erule subset_trans) | 
| 75 | apply (rule Abrial_axiom1) | |
| 76 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 77 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 78 | text{*Lemma 1 of section 3.1*}
 | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 79 | lemma TFin_linear_lemma1: | 
| 14706 | 80 | "[| n \<in> TFin S; m \<in> TFin S; | 
| 81 | \<forall>x \<in> TFin S. x \<subseteq> m --> x = m | succ S x \<subseteq> m | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 82 | |] ==> n \<subseteq> m | succ S m \<subseteq> n" | 
| 17200 | 83 | apply (erule TFin_induct) | 
| 84 | apply (erule_tac [2] Union_lemma0) | |
| 85 | apply (blast del: subsetI intro: succ_trans) | |
| 86 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 87 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 88 | text{* Lemma 2 of section 3.2 *}
 | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 89 | lemma TFin_linear_lemma2: | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 90 | "m \<in> TFin S ==> \<forall>n \<in> TFin S. n \<subseteq> m --> n=m | succ S n \<subseteq> m" | 
| 17200 | 91 | apply (erule TFin_induct) | 
| 92 | apply (rule impI [THEN ballI]) | |
| 93 |    txt{*case split using @{text TFin_linear_lemma1}*}
 | |
| 94 | apply (rule_tac n1 = n and m1 = x in TFin_linear_lemma1 [THEN disjE], | |
| 95 | assumption+) | |
| 96 | apply (drule_tac x = n in bspec, assumption) | |
| 97 | apply (blast del: subsetI intro: succ_trans, blast) | |
| 98 |   txt{*second induction step*}
 | |
| 99 | apply (rule impI [THEN ballI]) | |
| 100 | apply (rule Union_lemma0 [THEN disjE]) | |
| 101 | apply (rule_tac [3] disjI2) | |
| 102 | prefer 2 apply blast | |
| 103 | apply (rule ballI) | |
| 104 | apply (rule_tac n1 = n and m1 = x in TFin_linear_lemma1 [THEN disjE], | |
| 105 | assumption+, auto) | |
| 106 | apply (blast intro!: Abrial_axiom1 [THEN subsetD]) | |
| 107 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 108 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 109 | text{*Re-ordering the premises of Lemma 2*}
 | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 110 | lemma TFin_subsetD: | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 111 | "[| n \<subseteq> m; m \<in> TFin S; n \<in> TFin S |] ==> n=m | succ S n \<subseteq> m" | 
| 17200 | 112 | by (rule TFin_linear_lemma2 [rule_format]) | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 113 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 114 | text{*Consequences from section 3.3 -- Property 3.2, the ordering is total*}
 | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 115 | lemma TFin_subset_linear: "[| m \<in> TFin S; n \<in> TFin S|] ==> n \<subseteq> m | m \<subseteq> n" | 
| 17200 | 116 | apply (rule disjE) | 
| 117 | apply (rule TFin_linear_lemma1 [OF _ _TFin_linear_lemma2]) | |
| 118 | apply (assumption+, erule disjI2) | |
| 119 | apply (blast del: subsetI | |
| 120 | intro: subsetI Abrial_axiom1 [THEN subset_trans]) | |
| 121 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 122 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 123 | text{*Lemma 3 of section 3.3*}
 | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 124 | lemma eq_succ_upper: "[| n \<in> TFin S; m \<in> TFin S; m = succ S m |] ==> n \<subseteq> m" | 
| 17200 | 125 | apply (erule TFin_induct) | 
| 126 | apply (drule TFin_subsetD) | |
| 127 | apply (assumption+, force, blast) | |
| 128 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 129 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 130 | text{*Property 3.3 of section 3.3*}
 | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 131 | lemma equal_succ_Union: "m \<in> TFin S ==> (m = succ S m) = (m = Union(TFin S))" | 
| 17200 | 132 | apply (rule iffI) | 
| 133 | apply (rule Union_upper [THEN equalityI]) | |
| 18143 | 134 | apply assumption | 
| 135 | apply (rule eq_succ_upper [THEN Union_least], assumption+) | |
| 17200 | 136 | apply (erule ssubst) | 
| 137 | apply (rule Abrial_axiom1 [THEN equalityI]) | |
| 138 | apply (blast del: subsetI intro: subsetI TFin_UnionI TFin.succI) | |
| 139 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 140 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 141 | subsection{*Hausdorff's Theorem: Every Set Contains a Maximal Chain.*}
 | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 142 | |
| 14706 | 143 | text{*NB: We assume the partial ordering is @{text "\<subseteq>"},
 | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 144 | the subset relation!*} | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 145 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 146 | lemma empty_set_mem_chain: "({} :: 'a set set) \<in> chain S"
 | 
| 17200 | 147 | by (unfold chain_def) auto | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 148 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 149 | lemma super_subset_chain: "super S c \<subseteq> chain S" | 
| 17200 | 150 | by (unfold super_def) blast | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 151 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 152 | lemma maxchain_subset_chain: "maxchain S \<subseteq> chain S" | 
| 17200 | 153 | by (unfold maxchain_def) blast | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 154 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 155 | lemma mem_super_Ex: "c \<in> chain S - maxchain S ==> ? d. d \<in> super S c" | 
| 17200 | 156 | by (unfold super_def maxchain_def) auto | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 157 | |
| 18143 | 158 | lemma select_super: | 
| 159 | "c \<in> chain S - maxchain S ==> (\<some>c'. c': super S c): super S c" | |
| 17200 | 160 | apply (erule mem_super_Ex [THEN exE]) | 
| 161 | apply (rule someI2, auto) | |
| 162 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 163 | |
| 18143 | 164 | lemma select_not_equals: | 
| 165 | "c \<in> chain S - maxchain S ==> (\<some>c'. c': super S c) \<noteq> c" | |
| 17200 | 166 | apply (rule notI) | 
| 167 | apply (drule select_super) | |
| 168 | apply (simp add: super_def psubset_def) | |
| 169 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 170 | |
| 17200 | 171 | lemma succI3: "c \<in> chain S - maxchain S ==> succ S c = (\<some>c'. c': super S c)" | 
| 172 | by (unfold succ_def) (blast intro!: if_not_P) | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 173 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 174 | lemma succ_not_equals: "c \<in> chain S - maxchain S ==> succ S c \<noteq> c" | 
| 17200 | 175 | apply (frule succI3) | 
| 176 | apply (simp (no_asm_simp)) | |
| 177 | apply (rule select_not_equals, assumption) | |
| 178 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 179 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 180 | lemma TFin_chain_lemma4: "c \<in> TFin S ==> (c :: 'a set set): chain S" | 
| 17200 | 181 | apply (erule TFin_induct) | 
| 182 | apply (simp add: succ_def select_super [THEN super_subset_chain[THEN subsetD]]) | |
| 183 | apply (unfold chain_def) | |
| 184 | apply (rule CollectI, safe) | |
| 185 | apply (drule bspec, assumption) | |
| 186 | apply (rule_tac [2] m1 = Xa and n1 = X in TFin_subset_linear [THEN disjE], | |
| 187 | blast+) | |
| 188 | done | |
| 14706 | 189 | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 190 | theorem Hausdorff: "\<exists>c. (c :: 'a set set): maxchain S" | 
| 18143 | 191 | apply (rule_tac x = "Union (TFin S)" in exI) | 
| 17200 | 192 | apply (rule classical) | 
| 193 | apply (subgoal_tac "succ S (Union (TFin S)) = Union (TFin S) ") | |
| 194 | prefer 2 | |
| 195 | apply (blast intro!: TFin_UnionI equal_succ_Union [THEN iffD2, symmetric]) | |
| 196 | apply (cut_tac subset_refl [THEN TFin_UnionI, THEN TFin_chain_lemma4]) | |
| 197 | apply (drule DiffI [THEN succ_not_equals], blast+) | |
| 198 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 199 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 200 | |
| 14706 | 201 | subsection{*Zorn's Lemma: If All Chains Have Upper Bounds Then
 | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 202 | There Is a Maximal Element*} | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 203 | |
| 14706 | 204 | lemma chain_extend: | 
| 205 | "[| c \<in> chain S; z \<in> S; | |
| 18143 | 206 |         \<forall>x \<in> c. x \<subseteq> (z:: 'a set) |] ==> {z} Un c \<in> chain S"
 | 
| 17200 | 207 | by (unfold chain_def) blast | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 208 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 209 | lemma chain_Union_upper: "[| c \<in> chain S; x \<in> c |] ==> x \<subseteq> Union(c)" | 
| 17200 | 210 | by (unfold chain_def) auto | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 211 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 212 | lemma chain_ball_Union_upper: "c \<in> chain S ==> \<forall>x \<in> c. x \<subseteq> Union(c)" | 
| 17200 | 213 | by (unfold chain_def) auto | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 214 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 215 | lemma maxchain_Zorn: | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 216 | "[| c \<in> maxchain S; u \<in> S; Union(c) \<subseteq> u |] ==> Union(c) = u" | 
| 17200 | 217 | apply (rule ccontr) | 
| 218 | apply (simp add: maxchain_def) | |
| 219 | apply (erule conjE) | |
| 18143 | 220 |   apply (subgoal_tac "({u} Un c) \<in> super S c")
 | 
| 17200 | 221 | apply simp | 
| 222 | apply (unfold super_def psubset_def) | |
| 223 | apply (blast intro: chain_extend dest: chain_Union_upper) | |
| 224 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 225 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 226 | theorem Zorn_Lemma: | 
| 17200 | 227 | "\<forall>c \<in> chain S. Union(c): S ==> \<exists>y \<in> S. \<forall>z \<in> S. y \<subseteq> z --> y = z" | 
| 228 | apply (cut_tac Hausdorff maxchain_subset_chain) | |
| 229 | apply (erule exE) | |
| 230 | apply (drule subsetD, assumption) | |
| 231 | apply (drule bspec, assumption) | |
| 18143 | 232 | apply (rule_tac x = "Union(c)" in bexI) | 
| 17200 | 233 | apply (rule ballI, rule impI) | 
| 234 | apply (blast dest!: maxchain_Zorn, assumption) | |
| 235 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 236 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 237 | subsection{*Alternative version of Zorn's Lemma*}
 | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 238 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 239 | lemma Zorn_Lemma2: | 
| 17200 | 240 | "\<forall>c \<in> chain S. \<exists>y \<in> S. \<forall>x \<in> c. x \<subseteq> y | 
| 241 | ==> \<exists>y \<in> S. \<forall>x \<in> S. (y :: 'a set) \<subseteq> x --> y = x" | |
| 242 | apply (cut_tac Hausdorff maxchain_subset_chain) | |
| 243 | apply (erule exE) | |
| 244 | apply (drule subsetD, assumption) | |
| 245 | apply (drule bspec, assumption, erule bexE) | |
| 246 | apply (rule_tac x = y in bexI) | |
| 247 | prefer 2 apply assumption | |
| 248 | apply clarify | |
| 249 | apply (rule ccontr) | |
| 250 | apply (frule_tac z = x in chain_extend) | |
| 251 | apply (assumption, blast) | |
| 252 | apply (unfold maxchain_def super_def psubset_def) | |
| 253 | apply (blast elim!: equalityCE) | |
| 254 | done | |
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 255 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 256 | text{*Various other lemmas*}
 | 
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 257 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 258 | lemma chainD: "[| c \<in> chain S; x \<in> c; y \<in> c |] ==> x \<subseteq> y | y \<subseteq> x" | 
| 17200 | 259 | by (unfold chain_def) blast | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 260 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 261 | lemma chainD2: "!!(c :: 'a set set). c \<in> chain S ==> c \<subseteq> S" | 
| 17200 | 262 | by (unfold chain_def) blast | 
| 13551 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 263 | |
| 
b7f64ee8da84
converted Hyperreal/Zorn to Isar format and moved to Library
 paulson parents: diff
changeset | 264 | end |