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