prefer "locale begin ... end";
authorwenzelm
Wed, 29 Aug 2018 20:01:39 +0200
changeset 68847 511d163ab623
parent 68846 da0cb00a4d6a
child 68848 8825efd1c2cf
child 68849 0f9b2fa0556f
child 68890 725d5ed56563
prefer "locale begin ... end";
src/ZF/AC/AC16_WO4.thy
src/ZF/AC/DC.thy
--- a/src/ZF/AC/AC16_WO4.thy	Wed Aug 29 19:35:41 2018 +0200
+++ b/src/ZF/AC/AC16_WO4.thy	Wed Aug 29 20:01:39 2018 +0200
@@ -220,8 +220,9 @@
     and mpos[iff]:      "0<m"
     and Infinite[iff]:  "~ Finite(y)"
     and noLepoll:  "~ y \<lesssim> {v \<in> Pow(x). v \<approx> m}"
+begin
 
-lemma (in AC16) knat [iff]: "k \<in> nat"
+lemma knat [iff]: "k \<in> nat"
 by (simp add: k_def)
 
 
@@ -230,7 +231,7 @@
 (*      where a is certain k-2 element subset of y                        *)
 (* ********************************************************************** *)
 
-lemma (in AC16) Diff_Finite_eqpoll: "[| l \<approx> a; a \<subseteq> y |] ==> y - a \<approx> y"
+lemma Diff_Finite_eqpoll: "[| l \<approx> a; a \<subseteq> y |] ==> y - a \<approx> y"
 apply (insert WO_R Infinite lnat)
 apply (rule eqpoll_trans) 
 apply (rule Diff_lesspoll_eqpoll_Card) 
@@ -247,10 +248,10 @@
 done
 
 
-lemma (in AC16) s_subset: "s(u) \<subseteq> t_n"
+lemma s_subset: "s(u) \<subseteq> t_n"
 by (unfold s_def, blast)
 
-lemma (in AC16) sI: 
+lemma sI: 
       "[| w \<in> t_n; cons(b,cons(u,a)) \<subseteq> w; a \<subseteq> y; b \<in> y-a; l \<approx> a |] 
        ==> w \<in> s(u)"
 apply (unfold s_def succ_def k_def)
@@ -258,11 +259,11 @@
              intro: subset_imp_lepoll lepoll_trans)
 done
 
-lemma (in AC16) in_s_imp_u_in: "v \<in> s(u) ==> u \<in> v"
+lemma in_s_imp_u_in: "v \<in> s(u) ==> u \<in> v"
 by (unfold s_def, blast)
 
 
-lemma (in AC16) ex1_superset_a:
+lemma ex1_superset_a:
      "[| l \<approx> a;  a \<subseteq> y;  b \<in> y - a;  u \<in> x |]   
       ==> \<exists>! c. c \<in> s(u) & a \<subseteq> c & b \<in> c"
 apply (rule all_ex [simplified k_def, THEN ballE])
@@ -273,7 +274,7 @@
              intro!: cons_cons_subset eqpoll_sym [THEN cons_cons_eqpoll])
 done
 
-lemma (in AC16) the_eq_cons:
+lemma the_eq_cons:
      "[| \<forall>v \<in> s(u). succ(l) \<approx> v \<inter> y;   
          l \<approx> a;  a \<subseteq> y;  b \<in> y - a;  u \<in> x |]    
       ==> (THE c. c \<in> s(u) & a \<subseteq> c & b \<in> c) \<inter> y = cons(b, a)"
@@ -282,7 +283,7 @@
 apply (fast+)
 done
 
-lemma (in AC16) y_lepoll_subset_s:
+lemma y_lepoll_subset_s:
      "[| \<forall>v \<in> s(u). succ(l) \<approx> v \<inter> y;   
          l \<approx> a;  a \<subseteq> y;  u \<in> x |]   
       ==> y \<lesssim> {v \<in> s(u). a \<subseteq> v}"
@@ -306,14 +307,14 @@
 
 
 (*relies on the disjointness of x, y*)
-lemma (in AC16) x_imp_not_y [dest]: "a \<in> x ==> a \<notin> y"
+lemma x_imp_not_y [dest]: "a \<in> x ==> a \<notin> y"
 by (blast dest:  disjoint [THEN equalityD1, THEN subsetD, OF IntI])
 
-lemma (in AC16) w_Int_eq_w_Diff:
+lemma w_Int_eq_w_Diff:
      "w \<subseteq> x \<union> y ==> w \<inter> (x - {u}) = w - cons(u, w \<inter> y)" 
 by blast
 
-lemma (in AC16) w_Int_eqpoll_m:
+lemma w_Int_eqpoll_m:
      "[| w \<in> {v \<in> s(u). a \<subseteq> v};   
          l \<approx> a;  u \<in> x;   
          \<forall>v \<in> s(u). succ(l) \<approx> v \<inter> y |] 
@@ -335,12 +336,12 @@
 (*      to {v \<in> Pow(x). v \<approx> n-k}                                       *)
 (* ********************************************************************** *)
 
-lemma (in AC16) eqpoll_m_not_empty: "a \<approx> m ==> a \<noteq> 0"
+lemma eqpoll_m_not_empty: "a \<approx> m ==> a \<noteq> 0"
 apply (insert mpos)
 apply (fast elim!: zero_lt_natE dest!: eqpoll_succ_imp_not_empty)
 done
 
-lemma (in AC16) cons_cons_in:
+lemma cons_cons_in:
      "[| z \<in> xa \<inter> (x - {u}); l \<approx> a; a \<subseteq> y; u \<in> x |]   
       ==> \<exists>! w. w \<in> t_n & cons(z, cons(u, a)) \<subseteq> w"
 apply (rule all_ex [THEN bspec])
@@ -348,7 +349,7 @@
 apply (fast intro!: cons_eqpoll_succ elim: eqpoll_sym)
 done
 
-lemma (in AC16) subset_s_lepoll_w:
+lemma subset_s_lepoll_w:
      "[| \<forall>v \<in> s(u). succ(l) \<approx> v \<inter> y; a \<subseteq> y; l \<approx> a; u \<in> x |]   
       ==> {v \<in> s(u). a \<subseteq> v} \<lesssim> {v \<in> Pow(x). v \<approx> m}"
 apply (rule_tac f3 = "\<lambda>w \<in> {v \<in> s (u) . a \<subseteq> v}. w \<inter> (x - {u})" 
@@ -371,14 +372,14 @@
 (* well_ord_subsets_lepoll_n                                              *)
 (* ********************************************************************** *)
 
-lemma (in AC16) well_ord_subsets_eqpoll_n:
+lemma well_ord_subsets_eqpoll_n:
      "n \<in> nat ==> \<exists>S. well_ord({z \<in> Pow(y) . z \<approx> succ(n)}, S)"
 apply (rule WO_R [THEN well_ord_infinite_subsets_eqpoll_X,
                   THEN eqpoll_def [THEN def_imp_iff, THEN iffD1], THEN exE])
 apply (fast intro: bij_is_inj [THEN well_ord_rvimage])+
 done
 
-lemma (in AC16) well_ord_subsets_lepoll_n:
+lemma well_ord_subsets_lepoll_n:
      "n \<in> nat ==> \<exists>R. well_ord({z \<in> Pow(y). z \<lesssim> n}, R)"
 apply (induct_tac "n")
 apply (force intro!: well_ord_unit simp add: subsets_lepoll_0_eq_unit)
@@ -392,13 +393,13 @@
 done
 
 
-lemma (in AC16) LL_subset: "LL \<subseteq> {z \<in> Pow(y). z \<lesssim> succ(k #+ m)}"
+lemma LL_subset: "LL \<subseteq> {z \<in> Pow(y). z \<lesssim> succ(k #+ m)}"
 apply (unfold LL_def MM_def)
 apply (insert "includes")
 apply (blast intro: subset_imp_lepoll eqpoll_imp_lepoll lepoll_trans)
 done
 
-lemma (in AC16) well_ord_LL: "\<exists>S. well_ord(LL,S)"
+lemma well_ord_LL: "\<exists>S. well_ord(LL,S)"
 apply (rule well_ord_subsets_lepoll_n [THEN exE, of "succ(k#+m)"])
 apply simp 
 apply (blast intro: well_ord_subset [OF _ LL_subset])
@@ -408,7 +409,7 @@
 (* every element of LL is a contained in exactly one element of MM        *)
 (* ********************************************************************** *)
 
-lemma (in AC16) unique_superset_in_MM:
+lemma unique_superset_in_MM:
      "v \<in> LL ==> \<exists>! w. w \<in> MM & v \<subseteq> w"
 apply (unfold MM_def LL_def, safe, fast)
 apply (rule lepoll_imp_eqpoll_subset [THEN exE], assumption)
@@ -425,34 +426,34 @@
 (* The union of appropriate values is the whole x                         *)
 (* ********************************************************************** *)
 
-lemma (in AC16) Int_in_LL: "w \<in> MM ==> w \<inter> y \<in> LL"
+lemma Int_in_LL: "w \<in> MM ==> w \<inter> y \<in> LL"
 by (unfold LL_def, fast)
 
-lemma (in AC16) in_LL_eq_Int: 
+lemma in_LL_eq_Int: 
      "v \<in> LL ==> v = (THE x. x \<in> MM & v \<subseteq> x) \<inter> y"
 apply (unfold LL_def, clarify)
 apply (subst unique_superset_in_MM [THEN the_equality2])
 apply (auto simp add: Int_in_LL)
 done
 
-lemma (in AC16) unique_superset1: "a \<in> LL \<Longrightarrow> (THE x. x \<in> MM \<and> a \<subseteq> x) \<in> MM"
+lemma unique_superset1: "a \<in> LL \<Longrightarrow> (THE x. x \<in> MM \<and> a \<subseteq> x) \<in> MM"
 by (erule unique_superset_in_MM [THEN theI, THEN conjunct1]) 
 
-lemma (in AC16) the_in_MM_subset:
+lemma the_in_MM_subset:
      "v \<in> LL ==> (THE x. x \<in> MM & v \<subseteq> x) \<subseteq> x \<union> y"
 apply (drule unique_superset1)
 apply (unfold MM_def)
 apply (fast dest!: unique_superset1 "includes" [THEN subsetD])
 done
 
-lemma (in AC16) GG_subset: "v \<in> LL ==> GG ` v \<subseteq> x"
+lemma GG_subset: "v \<in> LL ==> GG ` v \<subseteq> x"
 apply (unfold GG_def)
 apply (frule the_in_MM_subset)
 apply (frule in_LL_eq_Int)
 apply (force elim: equalityE)
 done
 
-lemma (in AC16) nat_lepoll_ordertype: "nat \<lesssim> ordertype(y, R)"
+lemma nat_lepoll_ordertype: "nat \<lesssim> ordertype(y, R)"
 apply (rule nat_le_infinite_Ord [THEN le_imp_lepoll]) 
  apply (rule Ord_ordertype [OF WO_R]) 
 apply (rule ordertype_eqpoll [THEN eqpoll_imp_lepoll, THEN lepoll_infinite]) 
@@ -460,7 +461,7 @@
 apply (rule Infinite) 
 done
 
-lemma (in AC16) ex_subset_eqpoll_n: "n \<in> nat ==> \<exists>z. z \<subseteq> y & n \<approx> z"
+lemma ex_subset_eqpoll_n: "n \<in> nat ==> \<exists>z. z \<subseteq> y & n \<approx> z"
 apply (erule nat_lepoll_imp_ex_eqpoll_n)
 apply (rule lepoll_trans [OF nat_lepoll_ordertype]) 
 apply (rule ordertype_eqpoll [THEN eqpoll_sym, THEN eqpoll_imp_lepoll]) 
@@ -468,7 +469,7 @@
 done
 
 
-lemma (in AC16) exists_proper_in_s: "u \<in> x ==> \<exists>v \<in> s(u). succ(k) \<lesssim> v \<inter> y"
+lemma exists_proper_in_s: "u \<in> x ==> \<exists>v \<in> s(u). succ(k) \<lesssim> v \<inter> y"
 apply (rule ccontr)
 apply (subgoal_tac "\<forall>v \<in> s (u) . k \<approx> v \<inter> y")
 prefer 2 apply (simp add: s_def, blast intro: succ_not_lepoll_imp_eqpoll)
@@ -479,12 +480,12 @@
 apply (blast intro: lepoll_trans [OF y_lepoll_subset_s subset_s_lepoll_w])
 done
 
-lemma (in AC16) exists_in_MM: "u \<in> x ==> \<exists>w \<in> MM. u \<in> w"
+lemma exists_in_MM: "u \<in> x ==> \<exists>w \<in> MM. u \<in> w"
 apply (erule exists_proper_in_s [THEN bexE])
 apply (unfold MM_def s_def, fast)
 done
 
-lemma (in AC16) exists_in_LL: "u \<in> x ==> \<exists>w \<in> LL. u \<in> GG`w"
+lemma exists_in_LL: "u \<in> x ==> \<exists>w \<in> LL. u \<in> GG`w"
 apply (rule exists_in_MM [THEN bexE], assumption)
 apply (rule bexI)
 apply (erule_tac [2] Int_in_LL)
@@ -494,7 +495,7 @@
 apply (fast elim!: Int_in_LL)+
 done
 
-lemma (in AC16) OUN_eq_x: "well_ord(LL,S) ==>       
+lemma OUN_eq_x: "well_ord(LL,S) ==>       
       (\<Union>b<ordertype(LL,S). GG ` (converse(ordermap(LL,S)) ` b)) = x"
 apply (rule equalityI)
 apply (rule subsetI)
@@ -514,18 +515,18 @@
 (* Every element of the family is less than or equipollent to n-k (m)     *)
 (* ********************************************************************** *)
 
-lemma (in AC16) in_MM_eqpoll_n: "w \<in> MM ==> w \<approx> succ(k #+ m)"
+lemma in_MM_eqpoll_n: "w \<in> MM ==> w \<approx> succ(k #+ m)"
 apply (unfold MM_def)
 apply (fast dest: "includes" [THEN subsetD])
 done
 
-lemma (in AC16) in_LL_eqpoll_n: "w \<in> LL ==> succ(k) \<lesssim> w"
+lemma in_LL_eqpoll_n: "w \<in> LL ==> succ(k) \<lesssim> w"
 by (unfold LL_def MM_def, fast)
 
-lemma (in AC16) in_LL: "w \<in> LL ==> w \<subseteq> (THE x. x \<in> MM \<and> w \<subseteq> x)"
+lemma in_LL: "w \<in> LL ==> w \<subseteq> (THE x. x \<in> MM \<and> w \<subseteq> x)"
 by (erule subset_trans [OF in_LL_eq_Int [THEN equalityD1] Int_lower1])
 
-lemma (in AC16) all_in_lepoll_m: 
+lemma all_in_lepoll_m: 
       "well_ord(LL,S) ==>       
        \<forall>b<ordertype(LL,S). GG ` (converse(ordermap(LL,S)) ` b) \<lesssim> m"
 apply (unfold GG_def)
@@ -541,7 +542,7 @@
                                   THEN apply_type])+
 done
 
-lemma (in AC16) "conclusion":
+lemma "conclusion":
      "\<exists>a f. Ord(a) & domain(f) = a & (\<Union>b<a. f ` b) = x & (\<forall>b<a. f ` b \<lesssim> m)"
 apply (rule well_ord_LL [THEN exE])
 apply (rename_tac S)
@@ -553,13 +554,13 @@
                     Ord_ordertype  OUN_eq_x  all_in_lepoll_m [THEN ospec])
 done
 
+end
+
 
 (* ********************************************************************** *)
 (* The main theorem AC16(n, k) ==> WO4(n-k)                               *)
 (* ********************************************************************** *)
 
-term AC16
-
 theorem AC16_WO4: 
      "[| AC_Equiv.AC16(k #+ m, k); 0 < k; 0 < m; k \<in> nat; m \<in> nat |] ==> WO4(m)"
 apply (unfold AC_Equiv.AC16_def WO4_def)
--- a/src/ZF/AC/DC.thy	Wed Aug 29 19:35:41 2018 +0200
+++ b/src/ZF/AC/DC.thy	Wed Aug 29 20:01:39 2018 +0200
@@ -104,7 +104,7 @@
   defines XX_def: "XX == (\<Union>n \<in> nat. {f \<in> n->X. \<forall>k \<in> n. <f``k, f`k> \<in> R})"
      and RR_def:  "RR == {<z1,z2>:XX*XX. domain(z2)=succ(domain(z1))  
                                        & restrict(z2, domain(z1)) = z1}"
-
+begin
 
 (* ********************************************************************** *)
 (* DC ==> DC(omega)                                                       *)
@@ -132,10 +132,10 @@
 (*                                                                        *)
 (* ********************************************************************** *)
 
-lemma (in DC0_imp) lemma1_1: "RR \<subseteq> XX*XX"
+lemma lemma1_1: "RR \<subseteq> XX*XX"
 by (unfold RR_def, fast)
 
-lemma (in DC0_imp) lemma1_2: "RR \<noteq> 0"
+lemma lemma1_2: "RR \<noteq> 0"
 apply (unfold RR_def XX_def)
 apply (rule all_ex [THEN ballE])
 apply (erule_tac [2] notE [OF _ empty_subsetI [THEN PowI]])
@@ -152,7 +152,7 @@
 apply (simp add: singleton_0)
 done
 
-lemma (in DC0_imp) lemma1_3: "range(RR) \<subseteq> domain(RR)"
+lemma lemma1_3: "range(RR) \<subseteq> domain(RR)"
 apply (unfold RR_def XX_def)
 apply (rule range_subset_domain, blast, clarify)
 apply (frule fun_is_rel [THEN image_subset, THEN PowI, 
@@ -168,7 +168,7 @@
 apply (simp add: domain_of_fun succ_def restrict_cons_eq)
 done
 
-lemma (in DC0_imp) lemma2:
+lemma lemma2:
      "[| \<forall>n \<in> nat. <f`n, f`succ(n)> \<in> RR;  f \<in> nat -> XX;  n \<in> nat |]   
       ==> \<exists>k \<in> nat. f`succ(n) \<in> k -> X & n \<in> k   
                   & <f`succ(n)``n, f`succ(n)`n> \<in> R"
@@ -197,7 +197,7 @@
 apply (blast dest: domain_of_fun [symmetric, THEN trans] )
 done
 
-lemma (in DC0_imp) lemma3_1:
+lemma lemma3_1:
      "[| \<forall>n \<in> nat. <f`n, f`succ(n)> \<in> RR;  f \<in> nat -> XX;  m \<in> nat |]   
       ==>  {f`succ(x)`x. x \<in> m} = {f`succ(m)`x. x \<in> m}"
 apply (subgoal_tac "\<forall>x \<in> m. f`succ (m) `x = f`succ (x) `x")
@@ -220,7 +220,7 @@
              intro: nat_into_Ord OrdmemD [THEN subsetD])
 done
 
-lemma (in DC0_imp) lemma3:
+lemma lemma3:
      "[| \<forall>n \<in> nat. <f`n, f`succ(n)> \<in> RR;  f \<in> nat -> XX;  m \<in> nat |]  
       ==> (\<lambda>x \<in> nat. f`succ(x)`x) `` m = f`succ(m)``m"
 apply (erule natE, simp)
@@ -232,6 +232,7 @@
             elim!: image_fun [symmetric, OF _ OrdmemD [OF _ nat_into_Ord]])
 done
 
+end
 
 theorem DC0_imp_DC_nat: "DC0 ==> DC(nat)"
 apply (unfold DC_def DC0_def, clarify)
@@ -310,8 +311,9 @@
                     {<z1,z2>\<in>Fin(XX)*XX. (domain(z2)=succ(\<Union>f \<in> z1. domain(f))
                                     & (\<Union>f \<in> z1. domain(f)) = b  
                                     & (\<forall>f \<in> z1. restrict(z2,domain(f)) = f))}"
+begin
 
-lemma (in imp_DC0) lemma4:
+lemma lemma4:
      "[| range(R) \<subseteq> domain(R);  x \<in> domain(R) |]   
       ==> RR \<subseteq> Pow(XX)*XX &   
              (\<forall>Y \<in> Pow(XX). Y \<prec> nat \<longrightarrow> (\<exists>x \<in> XX. <Y,x>:RR))"
@@ -329,25 +331,25 @@
 apply (simp add: nat_0I [THEN rev_bexI] cons_fun_type2)
 done
 
-lemma (in imp_DC0) UN_image_succ_eq:
+lemma UN_image_succ_eq:
      "[| f \<in> nat->X; n \<in> nat |] 
       ==> (\<Union>x \<in> f``succ(n). P(x)) =  P(f`n) \<union> (\<Union>x \<in> f``n. P(x))"
 by (simp add: image_fun OrdmemD) 
 
-lemma (in imp_DC0) UN_image_succ_eq_succ:
+lemma UN_image_succ_eq_succ:
      "[| (\<Union>x \<in> f``n. P(x)) = y; P(f`n) = succ(y);   
          f \<in> nat -> X; n \<in> nat |] ==> (\<Union>x \<in> f``succ(n). P(x)) = succ(y)"
 by (simp add: UN_image_succ_eq, blast)
 
-lemma (in imp_DC0) apply_domain_type:
+lemma apply_domain_type:
      "[| h \<in> succ(n) -> D;  n \<in> nat; domain(h)=succ(y) |] ==> h`y \<in> D"
 by (fast elim: apply_type dest!: trans [OF sym domain_of_fun])
 
-lemma (in imp_DC0) image_fun_succ:
+lemma image_fun_succ:
      "[| h \<in> nat -> X; n \<in> nat |] ==> h``succ(n) = cons(h`n, h``n)"
 by (simp add: image_fun OrdmemD) 
 
-lemma (in imp_DC0) f_n_type:
+lemma f_n_type:
      "[| domain(f`n) = succ(k); f \<in> nat -> XX;  n \<in> nat |]    
       ==> f`n \<in> succ(k) -> domain(R)"
 apply (unfold XX_def)
@@ -355,7 +357,7 @@
 apply (fast elim: domain_eq_imp_fun_type)
 done
 
-lemma (in imp_DC0) f_n_pairs_in_R [rule_format]: 
+lemma f_n_pairs_in_R [rule_format]: 
      "[| h \<in> nat -> XX;  domain(h`n) = succ(k);  n \<in> nat |]   
       ==> \<forall>i \<in> k. <h`n`i, h`n`succ(i)> \<in> R"
 apply (unfold XX_def)
@@ -364,7 +366,7 @@
 apply (drule domain_of_fun [symmetric, THEN trans], assumption, simp)
 done
 
-lemma (in imp_DC0) restrict_cons_eq_restrict: 
+lemma restrict_cons_eq_restrict: 
      "[| restrict(h, domain(u))=u;  h \<in> n->X;  domain(u) \<subseteq> n |]   
       ==> restrict(cons(<n, y>, h), domain(u)) = u"
 apply (unfold restrict_def)
@@ -373,7 +375,7 @@
 apply (blast elim: mem_irrefl)  
 done
 
-lemma (in imp_DC0) all_in_image_restrict_eq:
+lemma all_in_image_restrict_eq:
      "[| \<forall>x \<in> f``n. restrict(f`n, domain(x))=x;   
          f \<in> nat -> XX;   
          n \<in> nat;  domain(f`n) = succ(n);   
@@ -387,7 +389,7 @@
 apply (blast intro!: restrict_cons_eq_restrict)
 done
 
-lemma (in imp_DC0) simplify_recursion: 
+lemma simplify_recursion: 
      "[| \<forall>b<nat. <f``b, f`b> \<in> RR;   
          f \<in> nat -> XX; range(R) \<subseteq> domain(R); x \<in> domain(R)|]    
       ==> allRR"
@@ -432,7 +434,7 @@
 done
 
 
-lemma (in imp_DC0) lemma2: 
+lemma lemma2: 
      "[| allRR; f \<in> nat->XX; range(R) \<subseteq> domain(R); x \<in> domain(R); n \<in> nat |]
       ==> f`n \<in> succ(n) -> domain(R) & (\<forall>i \<in> n. <f`n`i, f`n`succ(i)>:R)"
 apply (unfold allRR_def)
@@ -445,7 +447,7 @@
 apply (fast elim!: trans [THEN domain_eq_imp_fun_type] subst_context)
 done
 
-lemma (in imp_DC0) lemma3:
+lemma lemma3:
      "[| allRR; f \<in> nat->XX; n\<in>nat; range(R) \<subseteq> domain(R);  x \<in> domain(R) |]
       ==> f`n`n = f`succ(n)`n"
 apply (frule lemma2 [THEN conjunct1, THEN domain_of_fun], assumption+)
@@ -457,6 +459,8 @@
 apply (simp add: image_fun OrdmemD) 
 done
 
+end
+
 
 theorem DC_nat_imp_DC0: "DC(nat) ==> DC0"
 apply (unfold DC_def DC0_def)