src/ZF/AC/AC7_AC9.thy
author haftmann
Fri, 17 Jun 2005 16:12:49 +0200
changeset 16417 9bc16273c2d4
parent 14171 0cab06e3bbd0
child 27678 85ea2be46c71
permissions -rw-r--r--
migrated theory headers to new format
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
12787
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
     1
(*  Title:      ZF/AC/AC7_AC9.thy
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
     2
    ID:         $Id$
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
     3
    Author:     Krzysztof Grabczewski
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
     4
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
     5
The proofs needed to state that AC7, AC8 and AC9 are equivalent to the previous
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
     6
instances of AC.
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
     7
*)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
     8
16417
9bc16273c2d4 migrated theory headers to new format
haftmann
parents: 14171
diff changeset
     9
theory AC7_AC9 imports AC_Equiv begin
12787
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    10
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    11
(* ********************************************************************** *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    12
(* Lemmas used in the proofs AC7 ==> AC6 and AC9 ==> AC1                  *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    13
(*  - Sigma_fun_space_not0                                                *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    14
(*  - Sigma_fun_space_eqpoll                                              *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    15
(* ********************************************************************** *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    16
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    17
lemma Sigma_fun_space_not0: "[| 0\<notin>A; B \<in> A |] ==> (nat->Union(A)) * B \<noteq> 0"
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    18
by (blast dest!: Sigma_empty_iff [THEN iffD1] Union_empty_iff [THEN iffD1])
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    19
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    20
lemma inj_lemma: 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    21
        "C \<in> A ==> (\<lambda>g \<in> (nat->Union(A))*C.   
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    22
                (\<lambda>n \<in> nat. if(n=0, snd(g), fst(g)`(n #- 1))))   
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    23
                \<in> inj((nat->Union(A))*C, (nat->Union(A)) ) "
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    24
apply (unfold inj_def)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    25
apply (rule CollectI)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    26
apply (fast intro!: lam_type if_type apply_type fst_type snd_type, auto) 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    27
apply (rule fun_extension, assumption+)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    28
apply (drule lam_eqE [OF _ nat_succI], assumption, simp) 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    29
apply (drule lam_eqE [OF _ nat_0I], simp) 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    30
done
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    31
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    32
lemma Sigma_fun_space_eqpoll:
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    33
     "[| C \<in> A; 0\<notin>A |] ==> (nat->Union(A)) * C \<approx> (nat->Union(A))"
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    34
apply (rule eqpollI)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    35
apply (simp add: lepoll_def)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    36
apply (fast intro!: inj_lemma)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    37
apply (fast elim!: prod_lepoll_self not_sym [THEN not_emptyE] subst_elem 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    38
            elim: swap)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    39
done
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    40
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    41
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    42
(* ********************************************************************** *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    43
(* AC6 ==> AC7                                                            *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    44
(* ********************************************************************** *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    45
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    46
lemma AC6_AC7: "AC6 ==> AC7"
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    47
by (unfold AC6_def AC7_def, blast)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    48
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    49
(* ********************************************************************** *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    50
(* AC7 ==> AC6, Rubin & Rubin p. 12, Theorem 2.8                          *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    51
(* The case of the empty family of sets added in order to complete        *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    52
(* the proof.                                                             *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    53
(* ********************************************************************** *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    54
14171
0cab06e3bbd0 Extended the notion of letter and digit, such that now one may use greek,
skalberg
parents: 12787
diff changeset
    55
lemma lemma1_1: "y \<in> (\<Pi> B \<in> A. Y*B) ==> (\<lambda>B \<in> A. snd(y`B)) \<in> (\<Pi> B \<in> A. B)"
12787
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    56
by (fast intro!: lam_type snd_type apply_type)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    57
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    58
lemma lemma1_2:
14171
0cab06e3bbd0 Extended the notion of letter and digit, such that now one may use greek,
skalberg
parents: 12787
diff changeset
    59
     "y \<in> (\<Pi> B \<in> {Y*C. C \<in> A}. B) ==> (\<lambda>B \<in> A. y`(Y*B)) \<in> (\<Pi> B \<in> A. Y*B)"
12787
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    60
apply (fast intro!: lam_type apply_type)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    61
done
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    62
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    63
lemma AC7_AC6_lemma1:
14171
0cab06e3bbd0 Extended the notion of letter and digit, such that now one may use greek,
skalberg
parents: 12787
diff changeset
    64
     "(\<Pi> B \<in> {(nat->Union(A))*C. C \<in> A}. B) \<noteq> 0 ==> (\<Pi> B \<in> A. B) \<noteq> 0"
12787
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    65
by (fast intro!: equals0I lemma1_1 lemma1_2)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    66
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    67
lemma AC7_AC6_lemma2: "0 \<notin> A ==> 0 \<notin> {(nat -> Union(A)) * C. C \<in> A}"
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    68
by (blast dest: Sigma_fun_space_not0)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    69
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    70
lemma AC7_AC6: "AC7 ==> AC6"
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    71
apply (unfold AC6_def AC7_def)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    72
apply (rule allI)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    73
apply (rule impI)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    74
apply (case_tac "A=0", simp)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    75
apply (rule AC7_AC6_lemma1)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    76
apply (erule allE) 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    77
apply (blast del: notI
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    78
	     intro!: AC7_AC6_lemma2 intro: eqpoll_sym eqpoll_trans 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    79
                    Sigma_fun_space_eqpoll)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    80
done
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    81
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    82
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    83
(* ********************************************************************** *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    84
(* AC1 ==> AC8                                                            *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    85
(* ********************************************************************** *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    86
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    87
lemma AC1_AC8_lemma1: 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    88
        "\<forall>B \<in> A. \<exists>B1 B2. B=<B1,B2> & B1 \<approx> B2   
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    89
        ==> 0 \<notin> { bij(fst(B),snd(B)). B \<in> A }"
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    90
apply (unfold eqpoll_def, auto)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    91
done
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    92
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    93
lemma AC1_AC8_lemma2:
14171
0cab06e3bbd0 Extended the notion of letter and digit, such that now one may use greek,
skalberg
parents: 12787
diff changeset
    94
     "[| f \<in> (\<Pi> X \<in> RepFun(A,p). X); D \<in> A |] ==> (\<lambda>x \<in> A. f`p(x))`D \<in> p(D)" 
12787
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    95
apply (simp, fast elim!: apply_type)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    96
done
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    97
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    98
lemma AC1_AC8: "AC1 ==> AC8"
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
    99
apply (unfold AC1_def AC8_def)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   100
apply (fast dest: AC1_AC8_lemma1 AC1_AC8_lemma2)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   101
done
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   102
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   103
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   104
(* ********************************************************************** *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   105
(* AC8 ==> AC9                                                            *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   106
(*  - this proof replaces the following two from Rubin & Rubin:           *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   107
(*    AC8 ==> AC1 and AC1 ==> AC9                                         *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   108
(* ********************************************************************** *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   109
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   110
lemma AC8_AC9_lemma:
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   111
     "\<forall>B1 \<in> A. \<forall>B2 \<in> A. B1 \<approx> B2 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   112
      ==> \<forall>B \<in> A*A. \<exists>B1 B2. B=<B1,B2> & B1 \<approx> B2"
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   113
by fast
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   114
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   115
lemma AC8_AC9: "AC8 ==> AC9"
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   116
apply (unfold AC8_def AC9_def)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   117
apply (intro allI impI)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   118
apply (erule allE)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   119
apply (erule impE, erule AC8_AC9_lemma, force) 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   120
done
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   121
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   122
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   123
(* ********************************************************************** *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   124
(* AC9 ==> AC1                                                            *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   125
(* The idea of this proof comes from "Equivalents of the Axiom of Choice" *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   126
(* by Rubin & Rubin. But (x * y) is not necessarily equipollent to        *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   127
(* (x * y) Un {0} when y is a set of total functions acting from nat to   *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   128
(* Union(A) -- therefore we have used the set (y * nat) instead of y.     *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   129
(* ********************************************************************** *)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   130
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   131
lemma snd_lepoll_SigmaI: "b \<in> B \<Longrightarrow> X \<lesssim> B \<times> X"
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   132
by (blast intro: lepoll_trans prod_lepoll_self eqpoll_imp_lepoll 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   133
                 prod_commute_eqpoll) 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   134
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   135
lemma nat_lepoll_lemma:
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   136
     "[|0 \<notin> A; B \<in> A|] ==> nat \<lesssim> ((nat \<rightarrow> Union(A)) \<times> B) \<times> nat"
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   137
by (blast dest: Sigma_fun_space_not0 intro: snd_lepoll_SigmaI)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   138
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   139
lemma AC9_AC1_lemma1:
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   140
     "[| 0\<notin>A;  A\<noteq>0;   
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   141
         C = {((nat->Union(A))*B)*nat. B \<in> A}  Un  
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   142
             {cons(0,((nat->Union(A))*B)*nat). B \<in> A};  
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   143
         B1 \<in> C;  B2 \<in> C |]   
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   144
      ==> B1 \<approx> B2"
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   145
by (blast intro!: nat_lepoll_lemma Sigma_fun_space_eqpoll
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   146
                     nat_cons_eqpoll [THEN eqpoll_trans] 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   147
                     prod_eqpoll_cong [OF _ eqpoll_refl]
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   148
             intro: eqpoll_trans eqpoll_sym )
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   149
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   150
lemma AC9_AC1_lemma2:
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   151
     "\<forall>B1 \<in> {(F*B)*N. B \<in> A} Un {cons(0,(F*B)*N). B \<in> A}.   
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   152
      \<forall>B2 \<in> {(F*B)*N. B \<in> A} Un {cons(0,(F*B)*N). B \<in> A}.   
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   153
        f`<B1,B2> \<in> bij(B1, B2)   
14171
0cab06e3bbd0 Extended the notion of letter and digit, such that now one may use greek,
skalberg
parents: 12787
diff changeset
   154
      ==> (\<lambda>B \<in> A. snd(fst((f`<cons(0,(F*B)*N),(F*B)*N>)`0))) \<in> (\<Pi> X \<in> A. X)"
12787
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   155
apply (intro lam_type snd_type fst_type)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   156
apply (rule apply_type [OF _ consI1]) 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   157
apply (fast intro!: fun_weaken_type bij_is_fun)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   158
done
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   159
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   160
lemma AC9_AC1: "AC9 ==> AC1"
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   161
apply (unfold AC1_def AC9_def)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   162
apply (intro allI impI)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   163
apply (erule allE)
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   164
apply (case_tac "A~=0")
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   165
apply (blast dest: AC9_AC1_lemma1 AC9_AC1_lemma2, force) 
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   166
done
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   167
3ecbc37befab mistakenly deleted this theory
paulson
parents:
diff changeset
   168
end