src/ZF/Constructible/WF_absolute.thy
author paulson
Thu, 11 Jul 2002 17:18:28 +0200
changeset 13350 626b79677dfa
parent 13348 374d05460db4
child 13352 3cd767f8d78b
permissions -rw-r--r--
tidied
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
13306
6eebcddee32b more internalized formulas and separation proofs
paulson
parents: 13299
diff changeset
     1
header {*Absoluteness for Well-Founded Relations and Well-Founded Recursion*}
6eebcddee32b more internalized formulas and separation proofs
paulson
parents: 13299
diff changeset
     2
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
     3
theory WF_absolute = WFrec:
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
     4
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
     5
subsection{*Every well-founded relation is a subset of some inverse image of
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
     6
      an ordinal*}
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
     7
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
     8
lemma wf_rvimage_Ord: "Ord(i) \<Longrightarrow> wf(rvimage(A, f, Memrel(i)))"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
     9
by (blast intro: wf_rvimage wf_Memrel)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    10
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    11
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    12
constdefs
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    13
  wfrank :: "[i,i]=>i"
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    14
    "wfrank(r,a) == wfrec(r, a, %x f. \<Union>y \<in> r-``{x}. succ(f`y))"
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    15
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    16
constdefs
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    17
  wftype :: "i=>i"
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    18
    "wftype(r) == \<Union>y \<in> range(r). succ(wfrank(r,y))"
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    19
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    20
lemma wfrank: "wf(r) ==> wfrank(r,a) = (\<Union>y \<in> r-``{a}. succ(wfrank(r,y)))"
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    21
by (subst wfrank_def [THEN def_wfrec], simp_all)
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    22
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    23
lemma Ord_wfrank: "wf(r) ==> Ord(wfrank(r,a))"
13339
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
    24
apply (rule_tac a=a in wf_induct, assumption)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    25
apply (subst wfrank, assumption)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    26
apply (rule Ord_succ [THEN Ord_UN], blast)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    27
done
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    28
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    29
lemma wfrank_lt: "[|wf(r); <a,b> \<in> r|] ==> wfrank(r,a) < wfrank(r,b)"
13339
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
    30
apply (rule_tac a1 = b in wfrank [THEN ssubst], assumption)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    31
apply (rule UN_I [THEN ltI])
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    32
apply (simp add: Ord_wfrank vimage_iff)+
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    33
done
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    34
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    35
lemma Ord_wftype: "wf(r) ==> Ord(wftype(r))"
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    36
by (simp add: wftype_def Ord_wfrank)
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    37
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    38
lemma wftypeI: "\<lbrakk>wf(r);  x \<in> field(r)\<rbrakk> \<Longrightarrow> wfrank(r,x) \<in> wftype(r)"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    39
apply (simp add: wftype_def)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    40
apply (blast intro: wfrank_lt [THEN ltD])
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    41
done
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    42
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    43
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    44
lemma wf_imp_subset_rvimage:
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    45
     "[|wf(r); r \<subseteq> A*A|] ==> \<exists>i f. Ord(i) & r <= rvimage(A, f, Memrel(i))"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    46
apply (rule_tac x="wftype(r)" in exI)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    47
apply (rule_tac x="\<lambda>x\<in>A. wfrank(r,x)" in exI)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    48
apply (simp add: Ord_wftype, clarify)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    49
apply (frule subsetD, assumption, clarify)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    50
apply (simp add: rvimage_iff wfrank_lt [THEN ltD])
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    51
apply (blast intro: wftypeI)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    52
done
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    53
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    54
theorem wf_iff_subset_rvimage:
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    55
  "relation(r) ==> wf(r) <-> (\<exists>i f A. Ord(i) & r <= rvimage(A, f, Memrel(i)))"
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    56
by (blast dest!: relation_field_times_field wf_imp_subset_rvimage
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    57
          intro: wf_rvimage_Ord [THEN wf_subset])
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    58
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
    59
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    60
subsection{*Transitive closure without fixedpoints*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    61
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    62
constdefs
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    63
  rtrancl_alt :: "[i,i]=>i"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    64
    "rtrancl_alt(A,r) ==
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    65
       {p \<in> A*A. \<exists>n\<in>nat. \<exists>f \<in> succ(n) -> A.
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
    66
                 (\<exists>x y. p = <x,y> &  f`0 = x & f`n = y) &
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    67
                       (\<forall>i\<in>n. <f`i, f`succ(i)> \<in> r)}"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    68
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    69
lemma alt_rtrancl_lemma1 [rule_format]:
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    70
    "n \<in> nat
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    71
     ==> \<forall>f \<in> succ(n) -> field(r).
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    72
         (\<forall>i\<in>n. \<langle>f`i, f ` succ(i)\<rangle> \<in> r) --> \<langle>f`0, f`n\<rangle> \<in> r^*"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    73
apply (induct_tac n)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    74
apply (simp_all add: apply_funtype rtrancl_refl, clarify)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    75
apply (rename_tac n f)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    76
apply (rule rtrancl_into_rtrancl)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    77
 prefer 2 apply assumption
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    78
apply (drule_tac x="restrict(f,succ(n))" in bspec)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    79
 apply (blast intro: restrict_type2)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    80
apply (simp add: Ord_succ_mem_iff nat_0_le [THEN ltD] leI [THEN ltD] ltI)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    81
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    82
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    83
lemma rtrancl_alt_subset_rtrancl: "rtrancl_alt(field(r),r) <= r^*"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    84
apply (simp add: rtrancl_alt_def)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    85
apply (blast intro: alt_rtrancl_lemma1)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    86
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    87
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    88
lemma rtrancl_subset_rtrancl_alt: "r^* <= rtrancl_alt(field(r),r)"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    89
apply (simp add: rtrancl_alt_def, clarify)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    90
apply (frule rtrancl_type [THEN subsetD], clarify, simp)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    91
apply (erule rtrancl_induct)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    92
 txt{*Base case, trivial*}
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    93
 apply (rule_tac x=0 in bexI)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    94
  apply (rule_tac x="lam x:1. xa" in bexI)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    95
   apply simp_all
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    96
txt{*Inductive step*}
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    97
apply clarify
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    98
apply (rename_tac n f)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
    99
apply (rule_tac x="succ(n)" in bexI)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   100
 apply (rule_tac x="lam i:succ(succ(n)). if i=succ(n) then z else f`i" in bexI)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   101
  apply (simp add: Ord_succ_mem_iff nat_0_le [THEN ltD] leI [THEN ltD] ltI)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   102
  apply (blast intro: mem_asym)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   103
 apply typecheck
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   104
 apply auto
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   105
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   106
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   107
lemma rtrancl_alt_eq_rtrancl: "rtrancl_alt(field(r),r) = r^*"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   108
by (blast del: subsetI
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   109
	  intro: rtrancl_alt_subset_rtrancl rtrancl_subset_rtrancl_alt)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   110
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   111
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   112
constdefs
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   113
13324
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   114
  rtran_closure_mem :: "[i=>o,i,i,i] => o"
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   115
    --{*The property of belonging to @{text "rtran_closure(r)"}*}
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   116
    "rtran_closure_mem(M,A,r,p) ==
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   117
	      \<exists>nnat[M]. \<exists>n[M]. \<exists>n'[M]. 
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   118
               omega(M,nnat) & n\<in>nnat & successor(M,n,n') &
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   119
	       (\<exists>f[M]. typed_function(M,n',A,f) &
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   120
		(\<exists>x[M]. \<exists>y[M]. \<exists>zero[M]. pair(M,x,y,p) & empty(M,zero) &
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   121
		  fun_apply(M,f,zero,x) & fun_apply(M,f,n,y)) &
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   122
		  (\<forall>j[M]. j\<in>n --> 
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   123
		    (\<exists>fj[M]. \<exists>sj[M]. \<exists>fsj[M]. \<exists>ffp[M]. 
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   124
		      fun_apply(M,f,j,fj) & successor(M,j,sj) &
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   125
		      fun_apply(M,f,sj,fsj) & pair(M,fj,fsj,ffp) & ffp \<in> r)))"
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   126
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   127
  rtran_closure :: "[i=>o,i,i] => o"
13324
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   128
    "rtran_closure(M,r,s) == 
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   129
        \<forall>A[M]. is_field(M,r,A) -->
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   130
 	 (\<forall>p[M]. p \<in> s <-> rtran_closure_mem(M,A,r,p))"
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   131
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   132
  tran_closure :: "[i=>o,i,i] => o"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   133
    "tran_closure(M,r,t) ==
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   134
         \<exists>s[M]. rtran_closure(M,r,s) & composition(M,r,s,t)"
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   135
13324
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   136
lemma (in M_axioms) rtran_closure_mem_iff:
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   137
     "[|M(A); M(r); M(p)|]
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   138
      ==> rtran_closure_mem(M,A,r,p) <->
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   139
          (\<exists>n[M]. n\<in>nat & 
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   140
           (\<exists>f[M]. f \<in> succ(n) -> A &
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   141
            (\<exists>x[M]. \<exists>y[M]. p = <x,y> & f`0 = x & f`n = y) &
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   142
                           (\<forall>i\<in>n. <f`i, f`succ(i)> \<in> r)))"
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   143
apply (simp add: rtran_closure_mem_def typed_apply_abs
13339
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
   144
                 Ord_succ_mem_iff nat_0_le [THEN ltD], blast) 
13324
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   145
done
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   146
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   147
locale M_trancl = M_axioms +
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   148
  assumes rtrancl_separation:
13324
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   149
	 "[| M(r); M(A) |] ==> separation (M, rtran_closure_mem(M,A,r))"
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   150
      and wellfounded_trancl_separation:
13323
2c287f50c9f3 More relativization, reflection and proofs of separation
paulson
parents: 13306
diff changeset
   151
	 "[| M(r); M(Z) |] ==> 
2c287f50c9f3 More relativization, reflection and proofs of separation
paulson
parents: 13306
diff changeset
   152
	  separation (M, \<lambda>x. 
2c287f50c9f3 More relativization, reflection and proofs of separation
paulson
parents: 13306
diff changeset
   153
	      \<exists>w[M]. \<exists>wx[M]. \<exists>rp[M]. 
2c287f50c9f3 More relativization, reflection and proofs of separation
paulson
parents: 13306
diff changeset
   154
	       w \<in> Z & pair(M,w,x,wx) & tran_closure(M,r,rp) & wx \<in> rp)"
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   155
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   156
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   157
lemma (in M_trancl) rtran_closure_rtrancl:
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   158
     "M(r) ==> rtran_closure(M,r,rtrancl(r))"
13324
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   159
apply (simp add: rtran_closure_def rtran_closure_mem_iff 
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   160
                 rtrancl_alt_eq_rtrancl [symmetric] rtrancl_alt_def)
13339
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
   161
apply (auto simp add: nat_0_le [THEN ltD] apply_funtype) 
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   162
done
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   163
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   164
lemma (in M_trancl) rtrancl_closed [intro,simp]:
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   165
     "M(r) ==> M(rtrancl(r))"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   166
apply (insert rtrancl_separation [of r "field(r)"])
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   167
apply (simp add: rtrancl_alt_eq_rtrancl [symmetric]
13324
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   168
                 rtrancl_alt_def rtran_closure_mem_iff)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   169
done
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   170
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   171
lemma (in M_trancl) rtrancl_abs [simp]:
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   172
     "[| M(r); M(z) |] ==> rtran_closure(M,r,z) <-> z = rtrancl(r)"
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   173
apply (rule iffI)
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   174
 txt{*Proving the right-to-left implication*}
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   175
 prefer 2 apply (blast intro: rtran_closure_rtrancl)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   176
apply (rule M_equalityI)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   177
apply (simp add: rtran_closure_def rtrancl_alt_eq_rtrancl [symmetric]
13324
39d1b3a4c6f4 more and simpler separation proofs
paulson
parents: 13323
diff changeset
   178
                 rtrancl_alt_def rtran_closure_mem_iff)
13339
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
   179
apply (auto simp add: nat_0_le [THEN ltD] apply_funtype) 
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   180
done
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   181
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   182
lemma (in M_trancl) trancl_closed [intro,simp]:
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   183
     "M(r) ==> M(trancl(r))"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   184
by (simp add: trancl_def comp_closed rtrancl_closed)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   185
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   186
lemma (in M_trancl) trancl_abs [simp]:
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   187
     "[| M(r); M(z) |] ==> tran_closure(M,r,z) <-> z = trancl(r)"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   188
by (simp add: tran_closure_def trancl_def)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   189
13323
2c287f50c9f3 More relativization, reflection and proofs of separation
paulson
parents: 13306
diff changeset
   190
lemma (in M_trancl) wellfounded_trancl_separation':
2c287f50c9f3 More relativization, reflection and proofs of separation
paulson
parents: 13306
diff changeset
   191
     "[| M(r); M(Z) |] ==> separation (M, \<lambda>x. \<exists>w[M]. w \<in> Z & <w,x> \<in> r^+)"
2c287f50c9f3 More relativization, reflection and proofs of separation
paulson
parents: 13306
diff changeset
   192
by (insert wellfounded_trancl_separation [of r Z], simp) 
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   193
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   194
text{*Alternative proof of @{text wf_on_trancl}; inspiration for the
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   195
      relativized version.  Original version is on theory WF.*}
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   196
lemma "[| wf[A](r);  r-``A <= A |] ==> wf[A](r^+)"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   197
apply (simp add: wf_on_def wf_def)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   198
apply (safe intro!: equalityI)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   199
apply (drule_tac x = "{x\<in>A. \<exists>w. \<langle>w,x\<rangle> \<in> r^+ & w \<in> Z}" in spec)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   200
apply (blast elim: tranclE)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   201
done
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   202
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   203
lemma (in M_trancl) wellfounded_on_trancl:
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   204
     "[| wellfounded_on(M,A,r);  r-``A <= A; M(r); M(A) |]
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   205
      ==> wellfounded_on(M,A,r^+)"
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   206
apply (simp add: wellfounded_on_def)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   207
apply (safe intro!: equalityI)
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   208
apply (rename_tac Z x)
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   209
apply (subgoal_tac "M({x\<in>A. \<exists>w[M]. w \<in> Z & \<langle>w,x\<rangle> \<in> r^+})")
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   210
 prefer 2
13323
2c287f50c9f3 More relativization, reflection and proofs of separation
paulson
parents: 13306
diff changeset
   211
 apply (blast intro: wellfounded_trancl_separation') 
13299
3a932abf97e8 More use of relativized quantifiers
paulson
parents: 13293
diff changeset
   212
apply (drule_tac x = "{x\<in>A. \<exists>w[M]. w \<in> Z & \<langle>w,x\<rangle> \<in> r^+}" in rspec, safe)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   213
apply (blast dest: transM, simp)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   214
apply (rename_tac y w)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   215
apply (drule_tac x=w in bspec, assumption, clarify)
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   216
apply (erule tranclE)
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   217
  apply (blast dest: transM)   (*transM is needed to prove M(xa)*)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   218
 apply blast
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   219
done
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   220
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   221
lemma (in M_trancl) wellfounded_trancl:
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   222
     "[|wellfounded(M,r); M(r)|] ==> wellfounded(M,r^+)"
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   223
apply (rotate_tac -1)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   224
apply (simp add: wellfounded_iff_wellfounded_on_field)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   225
apply (rule wellfounded_on_subset_A, erule wellfounded_on_trancl)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   226
   apply blast
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   227
  apply (simp_all add: trancl_type [THEN field_rel_subset])
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   228
done
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   229
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   230
text{*Relativized to M: Every well-founded relation is a subset of some
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   231
inverse image of an ordinal.  Key step is the construction (in M) of a
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   232
rank function.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   233
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   234
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   235
locale M_wfrank = M_trancl +
13339
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
   236
  assumes wfrank_separation:
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   237
     "M(r) ==>
13339
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
   238
      separation (M, \<lambda>x. 
13348
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   239
         \<forall>rplus[M]. tran_closure(M,r,rplus) -->
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   240
         ~ (\<exists>f[M]. M_is_recfun(M, rplus, x, %x f y. is_range(M,f,y), f)))"
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   241
 and wfrank_strong_replacement:
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   242
     "M(r) ==>
13348
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   243
      strong_replacement(M, \<lambda>x z. 
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   244
         \<forall>rplus[M]. tran_closure(M,r,rplus) -->
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   245
         (\<exists>y[M]. \<exists>f[M]. pair(M,x,y,z)  & 
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   246
                        M_is_recfun(M, rplus, x, %x f y. is_range(M,f,y), f) &
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   247
                        is_range(M,f,y)))"
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   248
 and Ord_wfrank_separation:
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   249
     "M(r) ==>
13348
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   250
      separation (M, \<lambda>x.
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   251
         \<forall>rplus[M]. tran_closure(M,r,rplus) --> 
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   252
          ~ (\<forall>f[M]. \<forall>rangef[M]. 
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   253
             is_range(M,f,rangef) -->
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   254
             M_is_recfun(M, rplus, x, \<lambda>x f y. is_range(M,f,y), f) -->
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   255
             ordinal(M,rangef)))" 
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   256
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   257
text{*Proving that the relativized instances of Separation or Replacement
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   258
agree with the "real" ones.*}
13339
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
   259
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
   260
lemma (in M_wfrank) wfrank_separation':
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
   261
     "M(r) ==>
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
   262
      separation
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
   263
	   (M, \<lambda>x. ~ (\<exists>f[M]. is_recfun(r^+, x, %x f. range(f), f)))"
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
   264
apply (insert wfrank_separation [of r])
13350
paulson
parents: 13348
diff changeset
   265
apply (simp add: is_recfun_abs [of "%x. range"])
13339
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13324
diff changeset
   266
done
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   267
13348
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   268
lemma (in M_wfrank) wfrank_strong_replacement':
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   269
     "M(r) ==>
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   270
      strong_replacement(M, \<lambda>x z. \<exists>y[M]. \<exists>f[M]. 
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   271
		  pair(M,x,y,z) & is_recfun(r^+, x, %x f. range(f), f) &
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   272
		  y = range(f))"
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   273
apply (insert wfrank_strong_replacement [of r])
13350
paulson
parents: 13348
diff changeset
   274
apply (simp add: is_recfun_abs [of "%x. range"])
13348
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   275
done
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   276
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   277
lemma (in M_wfrank) Ord_wfrank_separation':
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   278
     "M(r) ==>
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   279
      separation (M, \<lambda>x. 
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   280
         ~ (\<forall>f[M]. is_recfun(r^+, x, \<lambda>x. range, f) --> Ord(range(f))))" 
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   281
apply (insert Ord_wfrank_separation [of r])
13350
paulson
parents: 13348
diff changeset
   282
apply (simp add: is_recfun_abs [of "%x. range"])
13348
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   283
done
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   284
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   285
text{*This function, defined using replacement, is a rank function for
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   286
well-founded relations within the class M.*}
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   287
constdefs
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   288
 wellfoundedrank :: "[i=>o,i,i] => i"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   289
    "wellfoundedrank(M,r,A) ==
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   290
        {p. x\<in>A, \<exists>y[M]. \<exists>f[M]. 
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   291
                       p = <x,y> & is_recfun(r^+, x, %x f. range(f), f) &
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   292
                       y = range(f)}"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   293
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   294
lemma (in M_wfrank) exists_wfrank:
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   295
    "[| wellfounded(M,r); M(a); M(r) |]
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   296
     ==> \<exists>f[M]. is_recfun(r^+, a, %x f. range(f), f)"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   297
apply (rule wellfounded_exists_is_recfun)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   298
      apply (blast intro: wellfounded_trancl)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   299
     apply (rule trans_trancl)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   300
    apply (erule wfrank_separation')
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   301
   apply (erule wfrank_strong_replacement')
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   302
apply (simp_all add: trancl_subset_times)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   303
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   304
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   305
lemma (in M_wfrank) M_wellfoundedrank:
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   306
    "[| wellfounded(M,r); M(r); M(A) |] ==> M(wellfoundedrank(M,r,A))"
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   307
apply (insert wfrank_strong_replacement' [of r])
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   308
apply (simp add: wellfoundedrank_def)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   309
apply (rule strong_replacement_closed)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   310
   apply assumption+
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   311
 apply (rule univalent_is_recfun)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   312
   apply (blast intro: wellfounded_trancl)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   313
  apply (rule trans_trancl)
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   314
 apply (simp add: trancl_subset_times, blast)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   315
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   316
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   317
lemma (in M_wfrank) Ord_wfrank_range [rule_format]:
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   318
    "[| wellfounded(M,r); a\<in>A; M(r); M(A) |]
13348
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   319
     ==> \<forall>f[M]. is_recfun(r^+, a, %x f. range(f), f) --> Ord(range(f))"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   320
apply (drule wellfounded_trancl, assumption)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   321
apply (rule wellfounded_induct, assumption+)
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   322
  apply simp
13348
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   323
 apply (blast intro: Ord_wfrank_separation', clarify)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   324
txt{*The reasoning in both cases is that we get @{term y} such that
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   325
   @{term "\<langle>y, x\<rangle> \<in> r^+"}.  We find that
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   326
   @{term "f`y = restrict(f, r^+ -`` {y})"}. *}
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   327
apply (rule OrdI [OF _ Ord_is_Transset])
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   328
 txt{*An ordinal is a transitive set...*}
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   329
 apply (simp add: Transset_def)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   330
 apply clarify
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   331
 apply (frule apply_recfun2, assumption)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   332
 apply (force simp add: restrict_iff)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   333
txt{*...of ordinals.  This second case requires the induction hyp.*}
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   334
apply clarify
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   335
apply (rename_tac i y)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   336
apply (frule apply_recfun2, assumption)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   337
apply (frule is_recfun_imp_in_r, assumption)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   338
apply (frule is_recfun_restrict)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   339
    (*simp_all won't work*)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   340
    apply (simp add: trans_trancl trancl_subset_times)+
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   341
apply (drule spec [THEN mp], assumption)
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   342
apply (subgoal_tac "M(restrict(f, r^+ -`` {y}))")
13348
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   343
 apply (drule_tac x="restrict(f, r^+ -`` {y})" in rspec)
374d05460db4 Separation/Replacement up to M_wfrank!
paulson
parents: 13339
diff changeset
   344
apply assumption
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   345
 apply (simp add: function_apply_equality [OF _ is_recfun_imp_function])
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   346
apply (blast dest: pair_components_in_M)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   347
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   348
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   349
lemma (in M_wfrank) Ord_range_wellfoundedrank:
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   350
    "[| wellfounded(M,r); r \<subseteq> A*A;  M(r); M(A) |]
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   351
     ==> Ord (range(wellfoundedrank(M,r,A)))"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   352
apply (frule wellfounded_trancl, assumption)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   353
apply (frule trancl_subset_times)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   354
apply (simp add: wellfoundedrank_def)
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   355
apply (rule OrdI [OF _ Ord_is_Transset])
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   356
 prefer 2
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   357
 txt{*by our previous result the range consists of ordinals.*}
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   358
 apply (blast intro: Ord_wfrank_range)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   359
txt{*We still must show that the range is a transitive set.*}
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   360
apply (simp add: Transset_def, clarify, simp)
13293
paulson
parents: 13269
diff changeset
   361
apply (rename_tac x i f u)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   362
apply (frule is_recfun_imp_in_r, assumption)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   363
apply (subgoal_tac "M(u) & M(i) & M(x)")
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   364
 prefer 2 apply (blast dest: transM, clarify)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   365
apply (rule_tac a=u in rangeI)
13293
paulson
parents: 13269
diff changeset
   366
apply (rule_tac x=u in ReplaceI)
paulson
parents: 13269
diff changeset
   367
  apply simp 
paulson
parents: 13269
diff changeset
   368
  apply (rule_tac x="restrict(f, r^+ -`` {u})" in rexI)
paulson
parents: 13269
diff changeset
   369
   apply (blast intro: is_recfun_restrict trans_trancl dest: apply_recfun2)
paulson
parents: 13269
diff changeset
   370
  apply simp 
paulson
parents: 13269
diff changeset
   371
apply blast 
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   372
txt{*Unicity requirement of Replacement*}
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   373
apply clarify
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   374
apply (frule apply_recfun2, assumption)
13293
paulson
parents: 13269
diff changeset
   375
apply (simp add: trans_trancl is_recfun_cut)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   376
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   377
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   378
lemma (in M_wfrank) function_wellfoundedrank:
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   379
    "[| wellfounded(M,r); M(r); M(A)|]
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   380
     ==> function(wellfoundedrank(M,r,A))"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   381
apply (simp add: wellfoundedrank_def function_def, clarify)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   382
txt{*Uniqueness: repeated below!*}
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   383
apply (drule is_recfun_functional, assumption)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   384
     apply (blast intro: wellfounded_trancl)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   385
    apply (simp_all add: trancl_subset_times trans_trancl)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   386
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   387
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   388
lemma (in M_wfrank) domain_wellfoundedrank:
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   389
    "[| wellfounded(M,r); M(r); M(A)|]
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   390
     ==> domain(wellfoundedrank(M,r,A)) = A"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   391
apply (simp add: wellfoundedrank_def function_def)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   392
apply (rule equalityI, auto)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   393
apply (frule transM, assumption)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   394
apply (frule_tac a=x in exists_wfrank, assumption+, clarify)
13293
paulson
parents: 13269
diff changeset
   395
apply (rule_tac b="range(f)" in domainI)
paulson
parents: 13269
diff changeset
   396
apply (rule_tac x=x in ReplaceI)
paulson
parents: 13269
diff changeset
   397
  apply simp 
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   398
  apply (rule_tac x=f in rexI, blast, simp_all)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   399
txt{*Uniqueness (for Replacement): repeated above!*}
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   400
apply clarify
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   401
apply (drule is_recfun_functional, assumption)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   402
    apply (blast intro: wellfounded_trancl)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   403
    apply (simp_all add: trancl_subset_times trans_trancl)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   404
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   405
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   406
lemma (in M_wfrank) wellfoundedrank_type:
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   407
    "[| wellfounded(M,r);  M(r); M(A)|]
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   408
     ==> wellfoundedrank(M,r,A) \<in> A -> range(wellfoundedrank(M,r,A))"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   409
apply (frule function_wellfoundedrank [of r A], assumption+)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   410
apply (frule function_imp_Pi)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   411
 apply (simp add: wellfoundedrank_def relation_def)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   412
 apply blast
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   413
apply (simp add: domain_wellfoundedrank)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   414
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   415
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   416
lemma (in M_wfrank) Ord_wellfoundedrank:
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   417
    "[| wellfounded(M,r); a \<in> A; r \<subseteq> A*A;  M(r); M(A) |]
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   418
     ==> Ord(wellfoundedrank(M,r,A) ` a)"
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   419
by (blast intro: apply_funtype [OF wellfoundedrank_type]
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   420
                 Ord_in_Ord [OF Ord_range_wellfoundedrank])
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   421
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   422
lemma (in M_wfrank) wellfoundedrank_eq:
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   423
     "[| is_recfun(r^+, a, %x. range, f);
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   424
         wellfounded(M,r);  a \<in> A; M(f); M(r); M(A)|]
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   425
      ==> wellfoundedrank(M,r,A) ` a = range(f)"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   426
apply (rule apply_equality)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   427
 prefer 2 apply (blast intro: wellfoundedrank_type)
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   428
apply (simp add: wellfoundedrank_def)
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   429
apply (rule ReplaceI)
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   430
  apply (rule_tac x="range(f)" in rexI) 
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   431
  apply blast
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   432
 apply simp_all
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   433
txt{*Unicity requirement of Replacement*}
13242
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   434
apply clarify
f96bd927dd37 towards absoluteness of wf
paulson
parents: 13223
diff changeset
   435
apply (drule is_recfun_functional, assumption)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   436
    apply (blast intro: wellfounded_trancl)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   437
    apply (simp_all add: trancl_subset_times trans_trancl)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   438
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   439
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   440
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   441
lemma (in M_wfrank) wellfoundedrank_lt:
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   442
     "[| <a,b> \<in> r;
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   443
         wellfounded(M,r); r \<subseteq> A*A;  M(r); M(A)|]
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   444
      ==> wellfoundedrank(M,r,A) ` a < wellfoundedrank(M,r,A) ` b"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   445
apply (frule wellfounded_trancl, assumption)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   446
apply (subgoal_tac "a\<in>A & b\<in>A")
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   447
 prefer 2 apply blast
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   448
apply (simp add: lt_def Ord_wellfoundedrank, clarify)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   449
apply (frule exists_wfrank [of concl: _ b], assumption+, clarify)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   450
apply (rename_tac fb)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   451
apply (frule is_recfun_restrict [of concl: "r^+" a])
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   452
    apply (rule trans_trancl, assumption)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   453
   apply (simp_all add: r_into_trancl trancl_subset_times)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   454
txt{*Still the same goal, but with new @{text is_recfun} assumptions.*}
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   455
apply (simp add: wellfoundedrank_eq)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   456
apply (frule_tac a=a in wellfoundedrank_eq, assumption+)
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   457
   apply (simp_all add: transM [of a])
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   458
txt{*We have used equations for wellfoundedrank and now must use some
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   459
    for  @{text is_recfun}. *}
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   460
apply (rule_tac a=a in rangeI)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   461
apply (simp add: is_recfun_type [THEN apply_iff] vimage_singleton_iff
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   462
                 r_into_trancl apply_recfun r_into_trancl)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   463
done
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   464
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   465
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   466
lemma (in M_wfrank) wellfounded_imp_subset_rvimage:
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   467
     "[|wellfounded(M,r); r \<subseteq> A*A; M(r); M(A)|]
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   468
      ==> \<exists>i f. Ord(i) & r <= rvimage(A, f, Memrel(i))"
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   469
apply (rule_tac x="range(wellfoundedrank(M,r,A))" in exI)
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   470
apply (rule_tac x="wellfoundedrank(M,r,A)" in exI)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   471
apply (simp add: Ord_range_wellfoundedrank, clarify)
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   472
apply (frule subsetD, assumption, clarify)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   473
apply (simp add: rvimage_iff wellfoundedrank_lt [THEN ltD])
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   474
apply (blast intro: apply_rangeI wellfoundedrank_type)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   475
done
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   476
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   477
lemma (in M_wfrank) wellfounded_imp_wf:
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   478
     "[|wellfounded(M,r); relation(r); M(r)|] ==> wf(r)"
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   479
by (blast dest!: relation_field_times_field wellfounded_imp_subset_rvimage
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   480
          intro: wf_rvimage_Ord [THEN wf_subset])
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   481
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   482
lemma (in M_wfrank) wellfounded_on_imp_wf_on:
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   483
     "[|wellfounded_on(M,A,r); relation(r); M(r); M(A)|] ==> wf[A](r)"
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   484
apply (simp add: wellfounded_on_iff_wellfounded wf_on_def)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   485
apply (rule wellfounded_imp_wf)
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   486
apply (simp_all add: relation_def)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   487
done
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   488
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   489
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   490
theorem (in M_wfrank) wf_abs [simp]:
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   491
     "[|relation(r); M(r)|] ==> wellfounded(M,r) <-> wf(r)"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   492
by (blast intro: wellfounded_imp_wf wf_imp_relativized)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   493
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   494
theorem (in M_wfrank) wf_on_abs [simp]:
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   495
     "[|relation(r); M(r); M(A)|] ==> wellfounded_on(M,A,r) <-> wf[A](r)"
13251
74cb2af8811e new treatment of wfrec, replacing wf[A](r) by wf(r)
paulson
parents: 13247
diff changeset
   496
by (blast intro: wellfounded_on_imp_wf_on wf_on_imp_relativized)
13247
e3c289f0724b towards absoluteness of wfrec-defined functions
paulson
parents: 13242
diff changeset
   497
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   498
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   499
text{*absoluteness for wfrec-defined functions.*}
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   500
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   501
(*first use is_recfun, then M_is_recfun*)
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   502
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   503
lemma (in M_trancl) wfrec_relativize:
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   504
  "[|wf(r); M(a); M(r);  
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   505
     strong_replacement(M, \<lambda>x z. \<exists>y[M]. \<exists>g[M].
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   506
          pair(M,x,y,z) & 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   507
          is_recfun(r^+, x, \<lambda>x f. H(x, restrict(f, r -`` {x})), g) & 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   508
          y = H(x, restrict(g, r -`` {x}))); 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   509
     \<forall>x[M]. \<forall>g[M]. function(g) --> M(H(x,g))|] 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   510
   ==> wfrec(r,a,H) = z <-> 
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   511
       (\<exists>f[M]. is_recfun(r^+, a, \<lambda>x f. H(x, restrict(f, r -`` {x})), f) & 
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   512
            z = H(a,restrict(f,r-``{a})))"
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   513
apply (frule wf_trancl) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   514
apply (simp add: wftrec_def wfrec_def, safe)
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   515
 apply (frule wf_exists_is_recfun 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   516
              [of concl: "r^+" a "\<lambda>x f. H(x, restrict(f, r -`` {x}))"]) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   517
      apply (simp_all add: trans_trancl function_restrictI trancl_subset_times)
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   518
 apply (clarify, rule_tac x=x in rexI) 
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   519
 apply (simp_all add: the_recfun_eq trans_trancl trancl_subset_times)
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   520
done
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   521
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   522
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   523
text{*Assuming @{term r} is transitive simplifies the occurrences of @{text H}.
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   524
      The premise @{term "relation(r)"} is necessary 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   525
      before we can replace @{term "r^+"} by @{term r}. *}
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   526
theorem (in M_trancl) trans_wfrec_relativize:
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   527
  "[|wf(r);  trans(r);  relation(r);  M(r);  M(a);
13293
paulson
parents: 13269
diff changeset
   528
     strong_replacement(M, \<lambda>x z. \<exists>y[M]. 
paulson
parents: 13269
diff changeset
   529
                pair(M,x,y,z) & (\<exists>g[M]. is_recfun(r,x,H,g) & y = H(x,g))); 
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   530
     \<forall>x[M]. \<forall>g[M]. function(g) --> M(H(x,g))|] 
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   531
   ==> wfrec(r,a,H) = z <-> (\<exists>f[M]. is_recfun(r,a,H,f) & z = H(a,f))" 
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   532
by (simp cong: is_recfun_cong
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   533
         add: wfrec_relativize trancl_eq_r
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   534
               is_recfun_restrict_idem domain_restrict_idem)
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   535
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   536
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   537
lemma (in M_trancl) trans_eq_pair_wfrec_iff:
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   538
  "[|wf(r);  trans(r); relation(r); M(r);  M(y); 
13293
paulson
parents: 13269
diff changeset
   539
     strong_replacement(M, \<lambda>x z. \<exists>y[M]. 
paulson
parents: 13269
diff changeset
   540
                pair(M,x,y,z) & (\<exists>g[M]. is_recfun(r,x,H,g) & y = H(x,g))); 
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   541
     \<forall>x[M]. \<forall>g[M]. function(g) --> M(H(x,g))|] 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   542
   ==> y = <x, wfrec(r, x, H)> <-> 
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   543
       (\<exists>f[M]. is_recfun(r,x,H,f) & y = <x, H(x,f)>)"
13293
paulson
parents: 13269
diff changeset
   544
apply safe 
paulson
parents: 13269
diff changeset
   545
 apply (simp add: trans_wfrec_relativize [THEN iff_sym, of concl: _ x]) 
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   546
txt{*converse direction*}
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   547
apply (rule sym)
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   548
apply (simp add: trans_wfrec_relativize, blast) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   549
done
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   550
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   551
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   552
subsection{*M is closed under well-founded recursion*}
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   553
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   554
text{*Lemma with the awkward premise mentioning @{text wfrec}.*}
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   555
lemma (in M_wfrank) wfrec_closed_lemma [rule_format]:
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   556
     "[|wf(r); M(r); 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   557
        strong_replacement(M, \<lambda>x y. y = \<langle>x, wfrec(r, x, H)\<rangle>);
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   558
        \<forall>x[M]. \<forall>g[M]. function(g) --> M(H(x,g)) |] 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   559
      ==> M(a) --> M(wfrec(r,a,H))"
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   560
apply (rule_tac a=a in wf_induct, assumption+)
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   561
apply (subst wfrec, assumption, clarify)
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   562
apply (drule_tac x1=x and x="\<lambda>x\<in>r -`` {x}. wfrec(r, x, H)" 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   563
       in rspec [THEN rspec]) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   564
apply (simp_all add: function_lam) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   565
apply (blast intro: dest: pair_components_in_M ) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   566
done
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   567
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   568
text{*Eliminates one instance of replacement.*}
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   569
lemma (in M_wfrank) wfrec_replacement_iff:
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   570
     "strong_replacement(M, \<lambda>x z. \<exists>y[M]. \<exists>g[M]. 
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   571
                pair(M,x,y,z) & is_recfun(r,x,H,g) & y = H(x,g)) <->
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   572
      strong_replacement(M, 
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   573
           \<lambda>x y. \<exists>f[M]. is_recfun(r,x,H,f) & y = <x, H(x,f)>)"
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   574
apply simp 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   575
apply (rule strong_replacement_cong, blast) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   576
done
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   577
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   578
text{*Useful version for transitive relations*}
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   579
theorem (in M_wfrank) trans_wfrec_closed:
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   580
     "[|wf(r); trans(r); relation(r); M(r); M(a);
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   581
        strong_replacement(M, 
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   582
             \<lambda>x z. \<exists>y[M]. \<exists>g[M].
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   583
                    pair(M,x,y,z) & is_recfun(r,x,H,g) & y = H(x,g)); 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   584
        \<forall>x[M]. \<forall>g[M]. function(g) --> M(H(x,g)) |] 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   585
      ==> M(wfrec(r,a,H))"
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   586
apply (frule wfrec_replacement_iff [THEN iffD1]) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   587
apply (rule wfrec_closed_lemma, assumption+) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   588
apply (simp_all add: wfrec_replacement_iff trans_eq_pair_wfrec_iff) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   589
done
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   590
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   591
section{*Absoluteness without assuming transitivity*}
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   592
lemma (in M_trancl) eq_pair_wfrec_iff:
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   593
  "[|wf(r);  M(r);  M(y); 
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   594
     strong_replacement(M, \<lambda>x z. \<exists>y[M]. \<exists>g[M].
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   595
          pair(M,x,y,z) & 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   596
          is_recfun(r^+, x, \<lambda>x f. H(x, restrict(f, r -`` {x})), g) & 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   597
          y = H(x, restrict(g, r -`` {x}))); 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   598
     \<forall>x[M]. \<forall>g[M]. function(g) --> M(H(x,g))|] 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   599
   ==> y = <x, wfrec(r, x, H)> <-> 
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   600
       (\<exists>f[M]. is_recfun(r^+, x, \<lambda>x f. H(x, restrict(f, r -`` {x})), f) & 
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   601
            y = <x, H(x,restrict(f,r-``{x}))>)"
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   602
apply safe  
13293
paulson
parents: 13269
diff changeset
   603
 apply (simp add: wfrec_relativize [THEN iff_sym, of concl: _ x]) 
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   604
txt{*converse direction*}
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   605
apply (rule sym)
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   606
apply (simp add: wfrec_relativize, blast) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   607
done
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   608
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   609
lemma (in M_wfrank) wfrec_closed_lemma [rule_format]:
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   610
     "[|wf(r); M(r); 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   611
        strong_replacement(M, \<lambda>x y. y = \<langle>x, wfrec(r, x, H)\<rangle>);
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   612
        \<forall>x[M]. \<forall>g[M]. function(g) --> M(H(x,g)) |] 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   613
      ==> M(a) --> M(wfrec(r,a,H))"
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   614
apply (rule_tac a=a in wf_induct, assumption+)
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   615
apply (subst wfrec, assumption, clarify)
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   616
apply (drule_tac x1=x and x="\<lambda>x\<in>r -`` {x}. wfrec(r, x, H)" 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   617
       in rspec [THEN rspec]) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   618
apply (simp_all add: function_lam) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   619
apply (blast intro: dest: pair_components_in_M ) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   620
done
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   621
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   622
text{*Full version not assuming transitivity, but maybe not very useful.*}
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   623
theorem (in M_wfrank) wfrec_closed:
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   624
     "[|wf(r); M(r); M(a);
13268
240509babf00 more use of relativized quantifiers
paulson
parents: 13254
diff changeset
   625
     strong_replacement(M, \<lambda>x z. \<exists>y[M]. \<exists>g[M].
13254
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   626
          pair(M,x,y,z) & 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   627
          is_recfun(r^+, x, \<lambda>x f. H(x, restrict(f, r -`` {x})), g) & 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   628
          y = H(x, restrict(g, r -`` {x}))); 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   629
        \<forall>x[M]. \<forall>g[M]. function(g) --> M(H(x,g)) |] 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   630
      ==> M(wfrec(r,a,H))"
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   631
apply (frule wfrec_replacement_iff [THEN iffD1]) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   632
apply (rule wfrec_closed_lemma, assumption+) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   633
apply (simp_all add: eq_pair_wfrec_iff) 
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   634
done
5146ccaedf42 class quantifiers (some)
paulson
parents: 13251
diff changeset
   635
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   636
end