src/ZF/Constructible/Normal.thy
author paulson
Tue, 06 Mar 2012 17:01:37 +0000
changeset 46823 57bf0cecb366
parent 32960 69916a850301
child 46927 faf4a0b02b71
permissions -rw-r--r--
More mathematical symbols for ZF examples
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
13505
52a16cb7fefb Relativized right up to L satisfies V=L!
paulson
parents: 13428
diff changeset
     1
(*  Title:      ZF/Constructible/Normal.thy
52a16cb7fefb Relativized right up to L satisfies V=L!
paulson
parents: 13428
diff changeset
     2
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
52a16cb7fefb Relativized right up to L satisfies V=L!
paulson
parents: 13428
diff changeset
     3
*)
52a16cb7fefb Relativized right up to L satisfies V=L!
paulson
parents: 13428
diff changeset
     4
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
     5
header {*Closed Unbounded Classes and Normal Functions*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
     6
16417
9bc16273c2d4 migrated theory headers to new format
haftmann
parents: 14171
diff changeset
     7
theory Normal imports Main begin
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
     8
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
     9
text{*
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    10
One source is the book
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    11
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    12
Frank R. Drake.
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    13
\emph{Set Theory: An Introduction to Large Cardinals}.
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    14
North-Holland, 1974.
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    15
*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    16
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    17
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    18
subsection {*Closed and Unbounded (c.u.) Classes of Ordinals*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    19
21233
5a5c8ea5f66a tuned specifications;
wenzelm
parents: 16417
diff changeset
    20
definition
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
    21
  Closed :: "(i=>o) => o" where
46823
57bf0cecb366 More mathematical symbols for ZF examples
paulson
parents: 32960
diff changeset
    22
    "Closed(P) == \<forall>I. I \<noteq> 0 \<longrightarrow> (\<forall>i\<in>I. Ord(i) \<and> P(i)) \<longrightarrow> P(\<Union>(I))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    23
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
    24
definition
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
    25
  Unbounded :: "(i=>o) => o" where
46823
57bf0cecb366 More mathematical symbols for ZF examples
paulson
parents: 32960
diff changeset
    26
    "Unbounded(P) == \<forall>i. Ord(i) \<longrightarrow> (\<exists>j. i<j \<and> P(j))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    27
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
    28
definition
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
    29
  Closed_Unbounded :: "(i=>o) => o" where
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    30
    "Closed_Unbounded(P) == Closed(P) \<and> Unbounded(P)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    31
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    32
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    33
subsubsection{*Simple facts about c.u. classes*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    34
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    35
lemma ClosedI:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    36
     "[| !!I. [| I \<noteq> 0; \<forall>i\<in>I. Ord(i) \<and> P(i) |] ==> P(\<Union>(I)) |] 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    37
      ==> Closed(P)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    38
by (simp add: Closed_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    39
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    40
lemma ClosedD:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    41
     "[| Closed(P); I \<noteq> 0; !!i. i\<in>I ==> Ord(i); !!i. i\<in>I ==> P(i) |] 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    42
      ==> P(\<Union>(I))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    43
by (simp add: Closed_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    44
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    45
lemma UnboundedD:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    46
     "[| Unbounded(P);  Ord(i) |] ==> \<exists>j. i<j \<and> P(j)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    47
by (simp add: Unbounded_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    48
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    49
lemma Closed_Unbounded_imp_Unbounded: "Closed_Unbounded(C) ==> Unbounded(C)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    50
by (simp add: Closed_Unbounded_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    51
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    52
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    53
text{*The universal class, V, is closed and unbounded.
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    54
      A bit odd, since C. U. concerns only ordinals, but it's used below!*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    55
theorem Closed_Unbounded_V [simp]: "Closed_Unbounded(\<lambda>x. True)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    56
by (unfold Closed_Unbounded_def Closed_def Unbounded_def, blast)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    57
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    58
text{*The class of ordinals, @{term Ord}, is closed and unbounded.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    59
theorem Closed_Unbounded_Ord   [simp]: "Closed_Unbounded(Ord)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    60
by (unfold Closed_Unbounded_def Closed_def Unbounded_def, blast)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    61
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    62
text{*The class of limit ordinals, @{term Limit}, is closed and unbounded.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    63
theorem Closed_Unbounded_Limit [simp]: "Closed_Unbounded(Limit)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    64
apply (simp add: Closed_Unbounded_def Closed_def Unbounded_def Limit_Union, 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    65
       clarify)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    66
apply (rule_tac x="i++nat" in exI)  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    67
apply (blast intro: oadd_lt_self oadd_LimitI Limit_nat Limit_has_0) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    68
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    69
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    70
text{*The class of cardinals, @{term Card}, is closed and unbounded.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    71
theorem Closed_Unbounded_Card  [simp]: "Closed_Unbounded(Card)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    72
apply (simp add: Closed_Unbounded_def Closed_def Unbounded_def Card_Union)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    73
apply (blast intro: lt_csucc Card_csucc)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    74
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    75
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    76
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    77
subsubsection{*The intersection of any set-indexed family of c.u. classes is
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    78
      c.u.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    79
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    80
text{*The constructions below come from Kunen, \emph{Set Theory}, page 78.*}
13428
99e52e78eb65 eliminate open locales and special ML code;
wenzelm
parents: 13382
diff changeset
    81
locale cub_family =
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    82
  fixes P and A
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    83
  fixes next_greater -- "the next ordinal satisfying class @{term A}"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    84
  fixes sup_greater  -- "sup of those ordinals over all @{term A}"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    85
  assumes closed:    "a\<in>A ==> Closed(P(a))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    86
      and unbounded: "a\<in>A ==> Unbounded(P(a))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    87
      and A_non0: "A\<noteq>0"
14171
0cab06e3bbd0 Extended the notion of letter and digit, such that now one may use greek,
skalberg
parents: 13634
diff changeset
    88
  defines "next_greater(a,x) == \<mu> y. x<y \<and> P(a,y)"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    89
      and "sup_greater(x) == \<Union>a\<in>A. next_greater(a,x)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    90
 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    91
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    92
text{*Trivial that the intersection is closed.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    93
lemma (in cub_family) Closed_INT: "Closed(\<lambda>x. \<forall>i\<in>A. P(i,x))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    94
by (blast intro: ClosedI ClosedD [OF closed])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    95
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    96
text{*All remaining effort goes to show that the intersection is unbounded.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    97
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    98
lemma (in cub_family) Ord_sup_greater:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    99
     "Ord(sup_greater(x))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   100
by (simp add: sup_greater_def next_greater_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   101
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   102
lemma (in cub_family) Ord_next_greater:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   103
     "Ord(next_greater(a,x))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   104
by (simp add: next_greater_def Ord_Least)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   105
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   106
text{*@{term next_greater} works as expected: it returns a larger value
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   107
and one that belongs to class @{term "P(a)"}. *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   108
lemma (in cub_family) next_greater_lemma:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   109
     "[| Ord(x); a\<in>A |] ==> P(a, next_greater(a,x)) \<and> x < next_greater(a,x)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   110
apply (simp add: next_greater_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   111
apply (rule exE [OF UnboundedD [OF unbounded]])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   112
  apply assumption+
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   113
apply (blast intro: LeastI2 lt_Ord2) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   114
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   115
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   116
lemma (in cub_family) next_greater_in_P:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   117
     "[| Ord(x); a\<in>A |] ==> P(a, next_greater(a,x))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   118
by (blast dest: next_greater_lemma)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   119
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   120
lemma (in cub_family) next_greater_gt:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   121
     "[| Ord(x); a\<in>A |] ==> x < next_greater(a,x)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   122
by (blast dest: next_greater_lemma)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   123
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   124
lemma (in cub_family) sup_greater_gt:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   125
     "Ord(x) ==> x < sup_greater(x)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   126
apply (simp add: sup_greater_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   127
apply (insert A_non0)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   128
apply (blast intro: UN_upper_lt next_greater_gt Ord_next_greater)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   129
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   130
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   131
lemma (in cub_family) next_greater_le_sup_greater:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   132
     "a\<in>A ==> next_greater(a,x) \<le> sup_greater(x)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   133
apply (simp add: sup_greater_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   134
apply (blast intro: UN_upper_le Ord_next_greater)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   135
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   136
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   137
lemma (in cub_family) omega_sup_greater_eq_UN:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   138
     "[| Ord(x); a\<in>A |] 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   139
      ==> sup_greater^\<omega> (x) = 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   140
          (\<Union>n\<in>nat. next_greater(a, sup_greater^n (x)))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   141
apply (simp add: iterates_omega_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   142
apply (rule le_anti_sym)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   143
apply (rule le_implies_UN_le_UN) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   144
apply (blast intro: leI next_greater_gt Ord_iterates Ord_sup_greater)  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   145
txt{*Opposite bound:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   146
@{subgoals[display,indent=0,margin=65]}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   147
*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   148
apply (rule UN_least_le) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   149
apply (blast intro: Ord_UN Ord_iterates Ord_sup_greater)  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   150
apply (rule_tac a="succ(n)" in UN_upper_le)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   151
apply (simp_all add: next_greater_le_sup_greater) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   152
apply (blast intro: Ord_UN Ord_iterates Ord_sup_greater)  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   153
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   154
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   155
lemma (in cub_family) P_omega_sup_greater:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   156
     "[| Ord(x); a\<in>A |] ==> P(a, sup_greater^\<omega> (x))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   157
apply (simp add: omega_sup_greater_eq_UN)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   158
apply (rule ClosedD [OF closed]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   159
apply (blast intro: ltD, auto)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   160
apply (blast intro: Ord_iterates Ord_next_greater Ord_sup_greater)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   161
apply (blast intro: next_greater_in_P Ord_iterates Ord_sup_greater)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   162
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   163
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   164
lemma (in cub_family) omega_sup_greater_gt:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   165
     "Ord(x) ==> x < sup_greater^\<omega> (x)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   166
apply (simp add: iterates_omega_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   167
apply (rule UN_upper_lt [of 1], simp_all) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   168
 apply (blast intro: sup_greater_gt) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   169
apply (blast intro: Ord_UN Ord_iterates Ord_sup_greater)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   170
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   171
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   172
lemma (in cub_family) Unbounded_INT: "Unbounded(\<lambda>x. \<forall>a\<in>A. P(a,x))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   173
apply (unfold Unbounded_def)  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   174
apply (blast intro!: omega_sup_greater_gt P_omega_sup_greater) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   175
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   176
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   177
lemma (in cub_family) Closed_Unbounded_INT: 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   178
     "Closed_Unbounded(\<lambda>x. \<forall>a\<in>A. P(a,x))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   179
by (simp add: Closed_Unbounded_def Closed_INT Unbounded_INT)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   180
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   181
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   182
theorem Closed_Unbounded_INT:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   183
    "(!!a. a\<in>A ==> Closed_Unbounded(P(a)))
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   184
     ==> Closed_Unbounded(\<lambda>x. \<forall>a\<in>A. P(a, x))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   185
apply (case_tac "A=0", simp)
13428
99e52e78eb65 eliminate open locales and special ML code;
wenzelm
parents: 13382
diff changeset
   186
apply (rule cub_family.Closed_Unbounded_INT [OF cub_family.intro])
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   187
apply (simp_all add: Closed_Unbounded_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   188
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   189
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   190
lemma Int_iff_INT2:
46823
57bf0cecb366 More mathematical symbols for ZF examples
paulson
parents: 32960
diff changeset
   191
     "P(x) \<and> Q(x)  \<longleftrightarrow>  (\<forall>i\<in>2. (i=0 \<longrightarrow> P(x)) \<and> (i=1 \<longrightarrow> Q(x)))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   192
by auto
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   193
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   194
theorem Closed_Unbounded_Int:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   195
     "[| Closed_Unbounded(P); Closed_Unbounded(Q) |] 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   196
      ==> Closed_Unbounded(\<lambda>x. P(x) \<and> Q(x))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   197
apply (simp only: Int_iff_INT2)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   198
apply (rule Closed_Unbounded_INT, auto) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   199
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   200
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   201
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   202
subsection {*Normal Functions*} 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   203
21233
5a5c8ea5f66a tuned specifications;
wenzelm
parents: 16417
diff changeset
   204
definition
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
   205
  mono_le_subset :: "(i=>i) => o" where
46823
57bf0cecb366 More mathematical symbols for ZF examples
paulson
parents: 32960
diff changeset
   206
    "mono_le_subset(M) == \<forall>i j. i\<le>j \<longrightarrow> M(i) \<subseteq> M(j)"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   207
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
   208
definition
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
   209
  mono_Ord :: "(i=>i) => o" where
46823
57bf0cecb366 More mathematical symbols for ZF examples
paulson
parents: 32960
diff changeset
   210
    "mono_Ord(F) == \<forall>i j. i<j \<longrightarrow> F(i) < F(j)"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   211
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
   212
definition
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
   213
  cont_Ord :: "(i=>i) => o" where
46823
57bf0cecb366 More mathematical symbols for ZF examples
paulson
parents: 32960
diff changeset
   214
    "cont_Ord(F) == \<forall>l. Limit(l) \<longrightarrow> F(l) = (\<Union>i<l. F(i))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   215
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
   216
definition
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
   217
  Normal :: "(i=>i) => o" where
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   218
    "Normal(F) == mono_Ord(F) \<and> cont_Ord(F)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   219
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   220
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   221
subsubsection{*Immediate properties of the definitions*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   222
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   223
lemma NormalI:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   224
     "[|!!i j. i<j ==> F(i) < F(j);  !!l. Limit(l) ==> F(l) = (\<Union>i<l. F(i))|]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   225
      ==> Normal(F)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   226
by (simp add: Normal_def mono_Ord_def cont_Ord_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   227
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   228
lemma mono_Ord_imp_Ord: "[| Ord(i); mono_Ord(F) |] ==> Ord(F(i))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   229
apply (simp add: mono_Ord_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   230
apply (blast intro: lt_Ord) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   231
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   232
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   233
lemma mono_Ord_imp_mono: "[| i<j; mono_Ord(F) |] ==> F(i) < F(j)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   234
by (simp add: mono_Ord_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   235
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   236
lemma Normal_imp_Ord [simp]: "[| Normal(F); Ord(i) |] ==> Ord(F(i))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   237
by (simp add: Normal_def mono_Ord_imp_Ord) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   238
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   239
lemma Normal_imp_cont: "[| Normal(F); Limit(l) |] ==> F(l) = (\<Union>i<l. F(i))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   240
by (simp add: Normal_def cont_Ord_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   241
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   242
lemma Normal_imp_mono: "[| i<j; Normal(F) |] ==> F(i) < F(j)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   243
by (simp add: Normal_def mono_Ord_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   244
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   245
lemma Normal_increasing: "[| Ord(i); Normal(F) |] ==> i\<le>F(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   246
apply (induct i rule: trans_induct3_rule)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   247
  apply (simp add: subset_imp_le)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   248
 apply (subgoal_tac "F(x) < F(succ(x))")
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   249
  apply (force intro: lt_trans1)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   250
 apply (simp add: Normal_def mono_Ord_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   251
apply (subgoal_tac "(\<Union>y<x. y) \<le> (\<Union>y<x. F(y))")
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   252
 apply (simp add: Normal_imp_cont Limit_OUN_eq) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   253
apply (blast intro: ltD le_implies_OUN_le_OUN)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   254
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   255
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   256
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   257
subsubsection{*The class of fixedpoints is closed and unbounded*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   258
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   259
text{*The proof is from Drake, pages 113--114.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   260
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   261
lemma mono_Ord_imp_le_subset: "mono_Ord(F) ==> mono_le_subset(F)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   262
apply (simp add: mono_le_subset_def, clarify)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   263
apply (subgoal_tac "F(i)\<le>F(j)", blast dest: le_imp_subset) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   264
apply (simp add: le_iff) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   265
apply (blast intro: lt_Ord2 mono_Ord_imp_Ord mono_Ord_imp_mono) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   266
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   267
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   268
text{*The following equation is taken for granted in any set theory text.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   269
lemma cont_Ord_Union:
46823
57bf0cecb366 More mathematical symbols for ZF examples
paulson
parents: 32960
diff changeset
   270
     "[| cont_Ord(F); mono_le_subset(F); X=0 \<longrightarrow> F(0)=0; \<forall>x\<in>X. Ord(x) |] 
57bf0cecb366 More mathematical symbols for ZF examples
paulson
parents: 32960
diff changeset
   271
      ==> F(\<Union>(X)) = (\<Union>y\<in>X. F(y))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   272
apply (frule Ord_set_cases)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   273
apply (erule disjE, force) 
46823
57bf0cecb366 More mathematical symbols for ZF examples
paulson
parents: 32960
diff changeset
   274
apply (thin_tac "X=0 \<longrightarrow> ?Q", auto)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   275
 txt{*The trival case of @{term "\<Union>X \<in> X"}*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   276
 apply (rule equalityI, blast intro: Ord_Union_eq_succD) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   277
 apply (simp add: mono_le_subset_def UN_subset_iff le_subset_iff) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   278
 apply (blast elim: equalityE)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   279
txt{*The limit case, @{term "Limit(\<Union>X)"}:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   280
@{subgoals[display,indent=0,margin=65]}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   281
*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   282
apply (simp add: OUN_Union_eq cont_Ord_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   283
apply (rule equalityI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   284
txt{*First inclusion:*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   285
 apply (rule UN_least [OF OUN_least])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   286
 apply (simp add: mono_le_subset_def, blast intro: leI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   287
txt{*Second inclusion:*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   288
apply (rule UN_least) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   289
apply (frule Union_upper_le, blast, blast intro: Ord_Union)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   290
apply (erule leE, drule ltD, elim UnionE)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   291
 apply (simp add: OUnion_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   292
 apply blast+
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   293
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   294
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   295
lemma Normal_Union:
46823
57bf0cecb366 More mathematical symbols for ZF examples
paulson
parents: 32960
diff changeset
   296
     "[| X\<noteq>0; \<forall>x\<in>X. Ord(x); Normal(F) |] ==> F(\<Union>(X)) = (\<Union>y\<in>X. F(y))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   297
apply (simp add: Normal_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   298
apply (blast intro: mono_Ord_imp_le_subset cont_Ord_Union) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   299
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   300
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   301
lemma Normal_imp_fp_Closed: "Normal(F) ==> Closed(\<lambda>i. F(i) = i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   302
apply (simp add: Closed_def ball_conj_distrib, clarify)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   303
apply (frule Ord_set_cases)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   304
apply (auto simp add: Normal_Union)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   305
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   306
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   307
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   308
lemma iterates_Normal_increasing:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   309
     "[| n\<in>nat;  x < F(x);  Normal(F) |] 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   310
      ==> F^n (x) < F^(succ(n)) (x)"  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   311
apply (induct n rule: nat_induct)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   312
apply (simp_all add: Normal_imp_mono)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   313
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   314
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   315
lemma Ord_iterates_Normal:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   316
     "[| n\<in>nat;  Normal(F);  Ord(x) |] ==> Ord(F^n (x))"  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   317
by (simp add: Ord_iterates) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   318
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   319
text{*THIS RESULT IS UNUSED*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   320
lemma iterates_omega_Limit:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   321
     "[| Normal(F);  x < F(x) |] ==> Limit(F^\<omega> (x))"  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   322
apply (frule lt_Ord) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   323
apply (simp add: iterates_omega_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   324
apply (rule increasing_LimitI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   325
   --"this lemma is @{thm increasing_LimitI [no_vars]}"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   326
 apply (blast intro: UN_upper_lt [of "1"]   Normal_imp_Ord
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   327
                     Ord_UN Ord_iterates lt_imp_0_lt
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13223
diff changeset
   328
                     iterates_Normal_increasing, clarify)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   329
apply (rule bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   330
 apply (blast intro: Ord_in_Ord [OF Ord_iterates_Normal]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   331
apply (rule UN_I, erule nat_succI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   332
apply (blast intro:  iterates_Normal_increasing Ord_iterates_Normal
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   333
                     ltD [OF lt_trans1, OF succ_leI, OF ltI]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   334
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   335
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   336
lemma iterates_omega_fixedpoint:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   337
     "[| Normal(F); Ord(a) |] ==> F(F^\<omega> (a)) = F^\<omega> (a)" 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   338
apply (frule Normal_increasing, assumption)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   339
apply (erule leE) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   340
 apply (simp_all add: iterates_omega_triv [OF sym])  (*for subgoal 2*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   341
apply (simp add:  iterates_omega_def Normal_Union) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   342
apply (rule equalityI, force simp add: nat_succI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   343
txt{*Opposite inclusion:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   344
@{subgoals[display,indent=0,margin=65]}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   345
*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   346
apply clarify
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   347
apply (rule UN_I, assumption) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   348
apply (frule iterates_Normal_increasing, assumption, assumption, simp)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   349
apply (blast intro: Ord_trans ltD Ord_iterates_Normal Normal_imp_Ord [of F]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   350
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   351
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   352
lemma iterates_omega_increasing:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   353
     "[| Normal(F); Ord(a) |] ==> a \<le> F^\<omega> (a)"   
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   354
apply (unfold iterates_omega_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   355
apply (rule UN_upper_le [of 0], simp_all)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   356
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   357
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   358
lemma Normal_imp_fp_Unbounded: "Normal(F) ==> Unbounded(\<lambda>i. F(i) = i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   359
apply (unfold Unbounded_def, clarify)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   360
apply (rule_tac x="F^\<omega> (succ(i))" in exI)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   361
apply (simp add: iterates_omega_fixedpoint) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   362
apply (blast intro: lt_trans2 [OF _ iterates_omega_increasing])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   363
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   364
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   365
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   366
theorem Normal_imp_fp_Closed_Unbounded: 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   367
     "Normal(F) ==> Closed_Unbounded(\<lambda>i. F(i) = i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   368
by (simp add: Closed_Unbounded_def Normal_imp_fp_Closed
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   369
              Normal_imp_fp_Unbounded)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   370
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   371
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   372
subsubsection{*Function @{text normalize}*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   373
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   374
text{*Function @{text normalize} maps a function @{text F} to a 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   375
      normal function that bounds it above.  The result is normal if and
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   376
      only if @{text F} is continuous: succ is not bounded above by any 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   377
      normal function, by @{thm [source] Normal_imp_fp_Unbounded}.
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   378
*}
21233
5a5c8ea5f66a tuned specifications;
wenzelm
parents: 16417
diff changeset
   379
definition
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
   380
  normalize :: "[i=>i, i] => i" where
46823
57bf0cecb366 More mathematical symbols for ZF examples
paulson
parents: 32960
diff changeset
   381
    "normalize(F,a) == transrec2(a, F(0), \<lambda>x r. F(succ(x)) \<union> succ(r))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   382
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   383
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   384
lemma Ord_normalize [simp, intro]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   385
     "[| Ord(a); !!x. Ord(x) ==> Ord(F(x)) |] ==> Ord(normalize(F, a))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   386
apply (induct a rule: trans_induct3_rule)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   387
apply (simp_all add: ltD def_transrec2 [OF normalize_def])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   388
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   389
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   390
lemma normalize_lemma [rule_format]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   391
     "[| Ord(b); !!x. Ord(x) ==> Ord(F(x)) |] 
46823
57bf0cecb366 More mathematical symbols for ZF examples
paulson
parents: 32960
diff changeset
   392
      ==> \<forall>a. a < b \<longrightarrow> normalize(F, a) < normalize(F, b)"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   393
apply (erule trans_induct3)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   394
  apply (simp_all add: le_iff def_transrec2 [OF normalize_def])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   395
 apply clarify
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   396
apply (rule Un_upper2_lt) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   397
  apply auto
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   398
 apply (drule spec, drule mp, assumption) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   399
 apply (erule leI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   400
apply (drule Limit_has_succ, assumption)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   401
apply (blast intro!: Ord_normalize intro: OUN_upper_lt ltD lt_Ord)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   402
done  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   403
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   404
lemma normalize_increasing:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   405
     "[| a < b;  !!x. Ord(x) ==> Ord(F(x)) |] 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   406
      ==> normalize(F, a) < normalize(F, b)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   407
by (blast intro!: normalize_lemma intro: lt_Ord2) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   408
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   409
theorem Normal_normalize:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   410
     "(!!x. Ord(x) ==> Ord(F(x))) ==> Normal(normalize(F))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   411
apply (rule NormalI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   412
apply (blast intro!: normalize_increasing)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   413
apply (simp add: def_transrec2 [OF normalize_def])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   414
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   415
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   416
theorem le_normalize:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   417
     "[| Ord(a); cont_Ord(F); !!x. Ord(x) ==> Ord(F(x)) |] 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   418
      ==> F(a) \<le> normalize(F,a)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   419
apply (erule trans_induct3) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   420
apply (simp_all add: def_transrec2 [OF normalize_def])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   421
apply (simp add: Un_upper1_le) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   422
apply (simp add: cont_Ord_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   423
apply (blast intro: ltD le_implies_OUN_le_OUN)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   424
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   425
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   426
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   427
subsection {*The Alephs*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   428
text {*This is the well-known transfinite enumeration of the cardinal 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   429
numbers.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   430
21233
5a5c8ea5f66a tuned specifications;
wenzelm
parents: 16417
diff changeset
   431
definition
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 21233
diff changeset
   432
  Aleph :: "i => i" where
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   433
    "Aleph(a) == transrec2(a, nat, \<lambda>x r. csucc(r))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   434
21233
5a5c8ea5f66a tuned specifications;
wenzelm
parents: 16417
diff changeset
   435
notation (xsymbols)
5a5c8ea5f66a tuned specifications;
wenzelm
parents: 16417
diff changeset
   436
  Aleph  ("\<aleph>_" [90] 90)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   437
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   438
lemma Card_Aleph [simp, intro]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   439
     "Ord(a) ==> Card(Aleph(a))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   440
apply (erule trans_induct3) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   441
apply (simp_all add: Card_csucc Card_nat Card_is_Ord
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   442
                     def_transrec2 [OF Aleph_def])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   443
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   444
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   445
lemma Aleph_lemma [rule_format]:
46823
57bf0cecb366 More mathematical symbols for ZF examples
paulson
parents: 32960
diff changeset
   446
     "Ord(b) ==> \<forall>a. a < b \<longrightarrow> Aleph(a) < Aleph(b)"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   447
apply (erule trans_induct3) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   448
apply (simp_all add: le_iff def_transrec2 [OF Aleph_def])  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   449
apply (blast intro: lt_trans lt_csucc Card_is_Ord, clarify)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   450
apply (drule Limit_has_succ, assumption)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   451
apply (blast intro: Card_is_Ord Card_Aleph OUN_upper_lt ltD lt_Ord)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   452
done  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   453
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   454
lemma Aleph_increasing:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   455
     "a < b ==> Aleph(a) < Aleph(b)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   456
by (blast intro!: Aleph_lemma intro: lt_Ord2) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   457
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   458
theorem Normal_Aleph: "Normal(Aleph)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   459
apply (rule NormalI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   460
apply (blast intro!: Aleph_increasing)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   461
apply (simp add: def_transrec2 [OF Aleph_def])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   462
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   463
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   464
end