src/ZF/Constructible/Reflection.thy
changeset 14171 0cab06e3bbd0
parent 13634 99a593b49b04
child 16417 9bc16273c2d4
equal deleted inserted replaced
14170:edd5a2ea3807 14171:0cab06e3bbd0
    40       and "Reflects(Cl,P,Q) == Closed_Unbounded(Cl) &
    40       and "Reflects(Cl,P,Q) == Closed_Unbounded(Cl) &
    41                               (\<forall>a. Cl(a) --> (\<forall>x\<in>Mset(a). P(x) <-> Q(a,x)))"
    41                               (\<forall>a. Cl(a) --> (\<forall>x\<in>Mset(a). P(x) <-> Q(a,x)))"
    42   fixes F0 --{*ordinal for a specific value @{term y}*}
    42   fixes F0 --{*ordinal for a specific value @{term y}*}
    43   fixes FF --{*sup over the whole level, @{term "y\<in>Mset(a)"}*}
    43   fixes FF --{*sup over the whole level, @{term "y\<in>Mset(a)"}*}
    44   fixes ClEx --{*Reflecting ordinals for the formula @{term "\<exists>z. P"}*}
    44   fixes ClEx --{*Reflecting ordinals for the formula @{term "\<exists>z. P"}*}
    45   defines "F0(P,y) == \<mu>b. (\<exists>z. M(z) & P(<y,z>)) --> 
    45   defines "F0(P,y) == \<mu> b. (\<exists>z. M(z) & P(<y,z>)) --> 
    46                                (\<exists>z\<in>Mset(b). P(<y,z>))"
    46                                (\<exists>z\<in>Mset(b). P(<y,z>))"
    47       and "FF(P)   == \<lambda>a. \<Union>y\<in>Mset(a). F0(P,y)"
    47       and "FF(P)   == \<lambda>a. \<Union>y\<in>Mset(a). F0(P,y)"
    48       and "ClEx(P,a) == Limit(a) & normalize(FF(P),a) = a"
    48       and "ClEx(P,a) == Limit(a) & normalize(FF(P),a) = a"
    49 
    49 
    50 lemma (in reflection) Mset_mono: "i\<le>j ==> Mset(i) <= Mset(j)"
    50 lemma (in reflection) Mset_mono: "i\<le>j ==> Mset(i) <= Mset(j)"
   352 
   352 
   353 text{*Example 4: Axiom of Choice.  Possibly wrong, since @{text \<Pi>} needs
   353 text{*Example 4: Axiom of Choice.  Possibly wrong, since @{text \<Pi>} needs
   354 to be relativized.*}
   354 to be relativized.*}
   355 lemma (in reflection) 
   355 lemma (in reflection) 
   356      "Reflects(?Cl,
   356      "Reflects(?Cl,
   357                \<lambda>A. 0\<notin>A --> (\<exists>f. M(f) & f \<in> (\<Pi>X \<in> A. X)),
   357                \<lambda>A. 0\<notin>A --> (\<exists>f. M(f) & f \<in> (\<Pi> X \<in> A. X)),
   358                \<lambda>a A. 0\<notin>A --> (\<exists>f\<in>Mset(a). f \<in> (\<Pi>X \<in> A. X)))"
   358                \<lambda>a A. 0\<notin>A --> (\<exists>f\<in>Mset(a). f \<in> (\<Pi> X \<in> A. X)))"
   359 by fast
   359 by fast
   360 
   360 
   361 end
   361 end
   362 
   362