src/ZF/Constructible/Formula.thy
author paulson
Wed, 21 Aug 2002 15:56:37 +0200
changeset 13511 e4b129eaa9c6
parent 13505 52a16cb7fefb
child 13535 007559e981c7
permissions -rw-r--r--
new proof needed now
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
13505
52a16cb7fefb Relativized right up to L satisfies V=L!
paulson
parents: 13398
diff changeset
     1
(*  Title:      ZF/Constructible/Formula.thy
52a16cb7fefb Relativized right up to L satisfies V=L!
paulson
parents: 13398
diff changeset
     2
    ID: $Id$
52a16cb7fefb Relativized right up to L satisfies V=L!
paulson
parents: 13398
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
52a16cb7fefb Relativized right up to L satisfies V=L!
paulson
parents: 13398
diff changeset
     4
    Copyright   2002  University of Cambridge
52a16cb7fefb Relativized right up to L satisfies V=L!
paulson
parents: 13398
diff changeset
     5
*)
52a16cb7fefb Relativized right up to L satisfies V=L!
paulson
parents: 13398
diff changeset
     6
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
     7
header {* First-Order Formulas and the Definition of the Class L *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
     8
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
     9
theory Formula = Main:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    10
13291
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
    11
subsection{*Internalized formulas of FOL*}
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
    12
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
    13
text{*De Bruijn representation.
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
    14
  Unbound variables get their denotations from an environment.*}
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    15
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    16
consts   formula :: i
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    17
datatype
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    18
  "formula" = Member ("x: nat", "y: nat")
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    19
            | Equal  ("x: nat", "y: nat")
13398
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    20
            | Nand ("p: formula", "q: formula")
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    21
            | Forall ("p: formula")
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    22
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    23
declare formula.intros [TC]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    24
13398
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    25
constdefs Neg :: "i=>i"
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    26
    "Neg(p) == Nand(p,p)"
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    27
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    28
constdefs And :: "[i,i]=>i"
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    29
    "And(p,q) == Neg(Nand(p,q))"
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    30
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    31
constdefs Or :: "[i,i]=>i"
13398
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    32
    "Or(p,q) == Nand(Neg(p),Neg(q))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    33
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    34
constdefs Implies :: "[i,i]=>i"
13398
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    35
    "Implies(p,q) == Nand(p,Neg(q))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    36
13291
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
    37
constdefs Iff :: "[i,i]=>i"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
    38
    "Iff(p,q) == And(Implies(p,q), Implies(q,p))"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
    39
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    40
constdefs Exists :: "i=>i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    41
    "Exists(p) == Neg(Forall(Neg(p)))";
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    42
13398
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    43
lemma Neg_type [TC]: "p \<in> formula ==> Neg(p) \<in> formula"
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    44
by (simp add: Neg_def) 
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    45
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    46
lemma And_type [TC]: "[| p \<in> formula; q \<in> formula |] ==> And(p,q) \<in> formula"
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    47
by (simp add: And_def) 
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    48
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    49
lemma Or_type [TC]: "[| p \<in> formula; q \<in> formula |] ==> Or(p,q) \<in> formula"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    50
by (simp add: Or_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    51
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    52
lemma Implies_type [TC]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    53
     "[| p \<in> formula; q \<in> formula |] ==> Implies(p,q) \<in> formula"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    54
by (simp add: Implies_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    55
13291
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
    56
lemma Iff_type [TC]:
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
    57
     "[| p \<in> formula; q \<in> formula |] ==> Iff(p,q) \<in> formula"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
    58
by (simp add: Iff_def) 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
    59
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    60
lemma Exists_type [TC]: "p \<in> formula ==> Exists(p) \<in> formula"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    61
by (simp add: Exists_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    62
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    63
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    64
consts   satisfies :: "[i,i]=>i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    65
primrec (*explicit lambda is required because the environment varies*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    66
  "satisfies(A,Member(x,y)) = 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    67
      (\<lambda>env \<in> list(A). bool_of_o (nth(x,env) \<in> nth(y,env)))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    68
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    69
  "satisfies(A,Equal(x,y)) = 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    70
      (\<lambda>env \<in> list(A). bool_of_o (nth(x,env) = nth(y,env)))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    71
13398
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    72
  "satisfies(A,Nand(p,q)) =
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    73
      (\<lambda>env \<in> list(A). not ((satisfies(A,p)`env) and (satisfies(A,q)`env)))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    74
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    75
  "satisfies(A,Forall(p)) = 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    76
      (\<lambda>env \<in> list(A). bool_of_o (\<forall>x\<in>A. satisfies(A,p) ` (Cons(x,env)) = 1))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    77
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    78
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    79
lemma "p \<in> formula ==> satisfies(A,p) \<in> list(A) -> bool"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    80
by (induct_tac p, simp_all) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    81
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    82
syntax sats :: "[i,i,i] => o"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    83
translations "sats(A,p,env)" == "satisfies(A,p)`env = 1"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    84
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    85
lemma [simp]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    86
  "env \<in> list(A) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    87
   ==> sats(A, Member(x,y), env) <-> nth(x,env) \<in> nth(y,env)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    88
by simp
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    89
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    90
lemma [simp]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    91
  "env \<in> list(A) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    92
   ==> sats(A, Equal(x,y), env) <-> nth(x,env) = nth(y,env)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    93
by simp
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    94
13398
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    95
lemma sats_Nand_iff [simp]:
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    96
  "env \<in> list(A) 
13398
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    97
   ==> (sats(A, Nand(p,q), env)) <-> ~ (sats(A,p,env) & sats(A,q,env))" 
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
    98
by (simp add: Bool.and_def Bool.not_def cond_def) 
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
    99
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   100
lemma sats_Forall_iff [simp]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   101
  "env \<in> list(A) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   102
   ==> sats(A, Forall(p), env) <-> (\<forall>x\<in>A. sats(A, p, Cons(x,env)))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   103
by simp
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   104
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   105
declare satisfies.simps [simp del]; 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   106
13298
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   107
subsection{*Dividing line between primitive and derived connectives*}
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   108
13398
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   109
lemma sats_Neg_iff [simp]:
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   110
  "env \<in> list(A) 
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   111
   ==> sats(A, Neg(p), env) <-> ~ sats(A,p,env)"
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   112
by (simp add: Neg_def) 
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   113
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   114
lemma sats_And_iff [simp]:
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   115
  "env \<in> list(A) 
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   116
   ==> (sats(A, And(p,q), env)) <-> sats(A,p,env) & sats(A,q,env)"
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   117
by (simp add: And_def) 
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   118
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   119
lemma sats_Or_iff [simp]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   120
  "env \<in> list(A) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   121
   ==> (sats(A, Or(p,q), env)) <-> sats(A,p,env) | sats(A,q,env)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   122
by (simp add: Or_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   123
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   124
lemma sats_Implies_iff [simp]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   125
  "env \<in> list(A) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   126
   ==> (sats(A, Implies(p,q), env)) <-> (sats(A,p,env) --> sats(A,q,env))"
13291
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   127
by (simp add: Implies_def, blast) 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   128
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   129
lemma sats_Iff_iff [simp]:
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   130
  "env \<in> list(A) 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   131
   ==> (sats(A, Iff(p,q), env)) <-> (sats(A,p,env) <-> sats(A,q,env))"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   132
by (simp add: Iff_def, blast) 
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   133
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   134
lemma sats_Exists_iff [simp]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   135
  "env \<in> list(A) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   136
   ==> sats(A, Exists(p), env) <-> (\<exists>x\<in>A. sats(A, p, Cons(x,env)))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   137
by (simp add: Exists_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   138
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   139
13291
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   140
subsubsection{*Derived rules to help build up formulas*}
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   141
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   142
lemma mem_iff_sats:
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   143
      "[| nth(i,env) = x; nth(j,env) = y; env \<in> list(A)|]
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   144
       ==> (x\<in>y) <-> sats(A, Member(i,j), env)" 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   145
by (simp add: satisfies.simps)
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   146
13298
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   147
lemma equal_iff_sats:
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   148
      "[| nth(i,env) = x; nth(j,env) = y; env \<in> list(A)|]
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   149
       ==> (x=y) <-> sats(A, Equal(i,j), env)" 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   150
by (simp add: satisfies.simps)
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   151
13316
d16629fd0f95 more and simpler separation proofs
paulson
parents: 13306
diff changeset
   152
lemma not_iff_sats:
d16629fd0f95 more and simpler separation proofs
paulson
parents: 13306
diff changeset
   153
      "[| P <-> sats(A,p,env); env \<in> list(A)|]
d16629fd0f95 more and simpler separation proofs
paulson
parents: 13306
diff changeset
   154
       ==> (~P) <-> sats(A, Neg(p), env)"
d16629fd0f95 more and simpler separation proofs
paulson
parents: 13306
diff changeset
   155
by simp
d16629fd0f95 more and simpler separation proofs
paulson
parents: 13306
diff changeset
   156
13291
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   157
lemma conj_iff_sats:
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   158
      "[| P <-> sats(A,p,env); Q <-> sats(A,q,env); env \<in> list(A)|]
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   159
       ==> (P & Q) <-> sats(A, And(p,q), env)"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   160
by (simp add: sats_And_iff)
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   161
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   162
lemma disj_iff_sats:
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   163
      "[| P <-> sats(A,p,env); Q <-> sats(A,q,env); env \<in> list(A)|]
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   164
       ==> (P | Q) <-> sats(A, Or(p,q), env)"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   165
by (simp add: sats_Or_iff)
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   166
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   167
lemma imp_iff_sats:
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   168
      "[| P <-> sats(A,p,env); Q <-> sats(A,q,env); env \<in> list(A)|]
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   169
       ==> (P --> Q) <-> sats(A, Implies(p,q), env)"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   170
by (simp add: sats_Forall_iff) 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   171
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   172
lemma iff_iff_sats:
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   173
      "[| P <-> sats(A,p,env); Q <-> sats(A,q,env); env \<in> list(A)|]
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   174
       ==> (P <-> Q) <-> sats(A, Iff(p,q), env)"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   175
by (simp add: sats_Forall_iff) 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   176
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   177
lemma imp_iff_sats:
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   178
      "[| P <-> sats(A,p,env); Q <-> sats(A,q,env); env \<in> list(A)|]
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   179
       ==> (P --> Q) <-> sats(A, Implies(p,q), env)"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   180
by (simp add: sats_Forall_iff) 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   181
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   182
lemma ball_iff_sats:
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   183
      "[| !!x. x\<in>A ==> P(x) <-> sats(A, p, Cons(x, env)); env \<in> list(A)|]
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   184
       ==> (\<forall>x\<in>A. P(x)) <-> sats(A, Forall(p), env)"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   185
by (simp add: sats_Forall_iff) 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   186
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   187
lemma bex_iff_sats:
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   188
      "[| !!x. x\<in>A ==> P(x) <-> sats(A, p, Cons(x, env)); env \<in> list(A)|]
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   189
       ==> (\<exists>x\<in>A. P(x)) <-> sats(A, Exists(p), env)"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   190
by (simp add: sats_Exists_iff) 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   191
13316
d16629fd0f95 more and simpler separation proofs
paulson
parents: 13306
diff changeset
   192
lemmas FOL_iff_sats = 
d16629fd0f95 more and simpler separation proofs
paulson
parents: 13306
diff changeset
   193
        mem_iff_sats equal_iff_sats not_iff_sats conj_iff_sats
d16629fd0f95 more and simpler separation proofs
paulson
parents: 13306
diff changeset
   194
        disj_iff_sats imp_iff_sats iff_iff_sats imp_iff_sats ball_iff_sats
d16629fd0f95 more and simpler separation proofs
paulson
parents: 13306
diff changeset
   195
        bex_iff_sats
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   196
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   197
constdefs incr_var :: "[i,i]=>i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   198
    "incr_var(x,lev) == if x<lev then x else succ(x)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   199
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   200
lemma incr_var_lt: "x<lev ==> incr_var(x,lev) = x"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   201
by (simp add: incr_var_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   202
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   203
lemma incr_var_le: "lev\<le>x ==> incr_var(x,lev) = succ(x)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   204
apply (simp add: incr_var_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   205
apply (blast dest: lt_trans1) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   206
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   207
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   208
consts   incr_bv :: "i=>i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   209
primrec
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   210
  "incr_bv(Member(x,y)) = 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   211
      (\<lambda>lev \<in> nat. Member (incr_var(x,lev), incr_var(y,lev)))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   212
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   213
  "incr_bv(Equal(x,y)) = 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   214
      (\<lambda>lev \<in> nat. Equal (incr_var(x,lev), incr_var(y,lev)))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   215
13398
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   216
  "incr_bv(Nand(p,q)) =
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   217
      (\<lambda>lev \<in> nat. Nand (incr_bv(p)`lev, incr_bv(q)`lev))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   218
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   219
  "incr_bv(Forall(p)) = 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   220
      (\<lambda>lev \<in> nat. Forall (incr_bv(p) ` succ(lev)))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   221
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   222
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   223
constdefs incr_boundvars :: "i => i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   224
    "incr_boundvars(p) == incr_bv(p)`0"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   225
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   226
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   227
lemma [TC]: "x \<in> nat ==> incr_var(x,lev) \<in> nat"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   228
by (simp add: incr_var_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   229
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   230
lemma incr_bv_type [TC]: "p \<in> formula ==> incr_bv(p) \<in> nat -> formula"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   231
by (induct_tac p, simp_all) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   232
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   233
lemma incr_boundvars_type [TC]: "p \<in> formula ==> incr_boundvars(p) \<in> formula"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   234
by (simp add: incr_boundvars_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   235
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   236
(*Obviously DPow is closed under complements and finite intersections and
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   237
unions.  Needs an inductive lemma to allow two lists of parameters to 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   238
be combined.*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   239
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   240
lemma sats_incr_bv_iff [rule_format]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   241
  "[| p \<in> formula; env \<in> list(A); x \<in> A |]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   242
   ==> \<forall>bvs \<in> list(A). 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   243
           sats(A, incr_bv(p) ` length(bvs), bvs @ Cons(x,env)) <-> 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   244
           sats(A, p, bvs@env)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   245
apply (induct_tac p)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   246
apply (simp_all add: incr_var_def nth_append succ_lt_iff length_type)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   247
apply (auto simp add: diff_succ not_lt_iff_le)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   248
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   249
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   250
(*UNUSED*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   251
lemma sats_incr_boundvars_iff:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   252
  "[| p \<in> formula; env \<in> list(A); x \<in> A |]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   253
   ==> sats(A, incr_boundvars(p), Cons(x,env)) <-> sats(A, p, env)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   254
apply (insert sats_incr_bv_iff [of p env A x Nil])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   255
apply (simp add: incr_boundvars_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   256
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   257
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   258
(*UNUSED
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   259
lemma formula_add_params [rule_format]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   260
  "[| p \<in> formula; n \<in> nat |]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   261
   ==> \<forall>bvs \<in> list(A). \<forall>env \<in> list(A). 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   262
         length(bvs) = n --> 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   263
         sats(A, iterates(incr_boundvars,n,p), bvs@env) <-> sats(A, p, env)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   264
apply (induct_tac n, simp, clarify) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   265
apply (erule list.cases)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   266
apply (auto simp add: sats_incr_boundvars_iff)  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   267
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   268
*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   269
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   270
consts   arity :: "i=>i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   271
primrec
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   272
  "arity(Member(x,y)) = succ(x) \<union> succ(y)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   273
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   274
  "arity(Equal(x,y)) = succ(x) \<union> succ(y)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   275
13398
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   276
  "arity(Nand(p,q)) = arity(p) \<union> arity(q)"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   277
13269
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   278
  "arity(Forall(p)) = nat_case(0, %x. x, arity(p))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   279
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   280
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   281
lemma arity_type [TC]: "p \<in> formula ==> arity(p) \<in> nat"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   282
by (induct_tac p, simp_all) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   283
13398
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   284
lemma arity_Neg [simp]: "arity(Neg(p)) = arity(p)"
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   285
by (simp add: Neg_def) 
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   286
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   287
lemma arity_And [simp]: "arity(And(p,q)) = arity(p) \<union> arity(q)"
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   288
by (simp add: And_def) 
1cadd412da48 Towards relativization and absoluteness of formula_rec
paulson
parents: 13385
diff changeset
   289
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   290
lemma arity_Or [simp]: "arity(Or(p,q)) = arity(p) \<union> arity(q)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   291
by (simp add: Or_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   292
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   293
lemma arity_Implies [simp]: "arity(Implies(p,q)) = arity(p) \<union> arity(q)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   294
by (simp add: Implies_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   295
13291
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   296
lemma arity_Iff [simp]: "arity(Iff(p,q)) = arity(p) \<union> arity(q)"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   297
by (simp add: Iff_def, blast)
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   298
13269
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   299
lemma arity_Exists [simp]: "arity(Exists(p)) = nat_case(0, %x. x, arity(p))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   300
by (simp add: Exists_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   301
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   302
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   303
lemma arity_sats_iff [rule_format]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   304
  "[| p \<in> formula; extra \<in> list(A) |]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   305
   ==> \<forall>env \<in> list(A). 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   306
           arity(p) \<le> length(env) --> 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   307
           sats(A, p, env @ extra) <-> sats(A, p, env)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   308
apply (induct_tac p)
13269
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   309
apply (simp_all add: nth_append Un_least_lt_iff arity_type nat_imp_quasinat
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   310
                split: split_nat_case, auto) 
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   311
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   312
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   313
lemma arity_sats1_iff:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   314
  "[| arity(p) \<le> succ(length(env)); p \<in> formula; x \<in> A; env \<in> list(A); 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   315
    extra \<in> list(A) |]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   316
   ==> sats(A, p, Cons(x, env @ extra)) <-> sats(A, p, Cons(x, env))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   317
apply (insert arity_sats_iff [of p extra A "Cons(x,env)"])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   318
apply simp 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   319
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   320
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   321
(*the following two lemmas prevent huge case splits in arity_incr_bv_lemma*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   322
lemma incr_var_lemma:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   323
     "[| x \<in> nat; y \<in> nat; lev \<le> x |]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   324
      ==> succ(x) \<union> incr_var(y,lev) = succ(x \<union> y)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   325
apply (simp add: incr_var_def Ord_Un_if, auto)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   326
  apply (blast intro: leI)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   327
 apply (simp add: not_lt_iff_le)  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   328
 apply (blast intro: le_anti_sym) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   329
apply (blast dest: lt_trans2) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   330
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   331
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   332
lemma incr_And_lemma:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   333
     "y < x ==> y \<union> succ(x) = succ(x \<union> y)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   334
apply (simp add: Ord_Un_if lt_Ord lt_Ord2 succ_lt_iff) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   335
apply (blast dest: lt_asym) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   336
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   337
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   338
lemma arity_incr_bv_lemma [rule_format]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   339
  "p \<in> formula 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   340
   ==> \<forall>n \<in> nat. arity (incr_bv(p) ` n) = 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   341
                 (if n < arity(p) then succ(arity(p)) else arity(p))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   342
apply (induct_tac p) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   343
apply (simp_all add: imp_disj not_lt_iff_le Un_least_lt_iff lt_Un_iff le_Un_iff
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   344
                     succ_Un_distrib [symmetric] incr_var_lt incr_var_le
13269
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   345
                     Un_commute incr_var_lemma arity_type nat_imp_quasinat
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   346
            split: split_nat_case) 
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   347
 txt{*the Forall case reduces to linear arithmetic*}
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   348
 prefer 2
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   349
 apply clarify 
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   350
 apply (blast dest: lt_trans1) 
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   351
txt{*left with the And case*}
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   352
apply safe
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   353
 apply (blast intro: incr_And_lemma lt_trans1) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   354
apply (subst incr_And_lemma)
13269
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   355
 apply (blast intro: lt_trans1) 
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   356
apply (simp add: Un_commute)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   357
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   358
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   359
lemma arity_incr_boundvars_eq:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   360
  "p \<in> formula
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   361
   ==> arity(incr_boundvars(p)) =
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   362
        (if 0 < arity(p) then succ(arity(p)) else arity(p))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   363
apply (insert arity_incr_bv_lemma [of p 0])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   364
apply (simp add: incr_boundvars_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   365
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   366
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   367
lemma arity_iterates_incr_boundvars_eq:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   368
  "[| p \<in> formula; n \<in> nat |]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   369
   ==> arity(incr_boundvars^n(p)) =
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   370
         (if 0 < arity(p) then n #+ arity(p) else arity(p))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   371
apply (induct_tac n) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   372
apply (simp_all add: arity_incr_boundvars_eq not_lt_iff_le) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   373
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   374
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   375
13298
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   376
subsection{*Renaming all but the first bound variable*}
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   377
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   378
constdefs incr_bv1 :: "i => i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   379
    "incr_bv1(p) == incr_bv(p)`1"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   380
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   381
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   382
lemma incr_bv1_type [TC]: "p \<in> formula ==> incr_bv1(p) \<in> formula"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   383
by (simp add: incr_bv1_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   384
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   385
(*For renaming all but the bound variable at level 0*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   386
lemma sats_incr_bv1_iff [rule_format]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   387
  "[| p \<in> formula; env \<in> list(A); x \<in> A; y \<in> A |]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   388
   ==> sats(A, incr_bv1(p), Cons(x, Cons(y, env))) <-> 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   389
       sats(A, p, Cons(x,env))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   390
apply (insert sats_incr_bv_iff [of p env A y "Cons(x,Nil)"])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   391
apply (simp add: incr_bv1_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   392
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   393
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   394
lemma formula_add_params1 [rule_format]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   395
  "[| p \<in> formula; n \<in> nat; x \<in> A |]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   396
   ==> \<forall>bvs \<in> list(A). \<forall>env \<in> list(A). 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   397
          length(bvs) = n --> 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   398
          sats(A, iterates(incr_bv1, n, p), Cons(x, bvs@env)) <-> 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   399
          sats(A, p, Cons(x,env))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   400
apply (induct_tac n, simp, clarify) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   401
apply (erule list.cases)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   402
apply (simp_all add: sats_incr_bv1_iff) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   403
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   404
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   405
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   406
lemma arity_incr_bv1_eq:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   407
  "p \<in> formula
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   408
   ==> arity(incr_bv1(p)) =
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   409
        (if 1 < arity(p) then succ(arity(p)) else arity(p))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   410
apply (insert arity_incr_bv_lemma [of p 1])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   411
apply (simp add: incr_bv1_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   412
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   413
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   414
lemma arity_iterates_incr_bv1_eq:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   415
  "[| p \<in> formula; n \<in> nat |]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   416
   ==> arity(incr_bv1^n(p)) =
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   417
         (if 1 < arity(p) then n #+ arity(p) else arity(p))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   418
apply (induct_tac n) 
13298
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   419
apply (simp_all add: arity_incr_bv1_eq)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   420
apply (simp add: not_lt_iff_le)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   421
apply (blast intro: le_trans add_le_self2 arity_type) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   422
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   423
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   424
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   425
(*Definable powerset operation: Kunen's definition 1.1, page 165.*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   426
constdefs DPow :: "i => i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   427
  "DPow(A) == {X \<in> Pow(A). 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   428
               \<exists>env \<in> list(A). \<exists>p \<in> formula. 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   429
                 arity(p) \<le> succ(length(env)) & 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   430
                 X = {x\<in>A. sats(A, p, Cons(x,env))}}"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   431
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   432
lemma DPowI:
13291
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   433
  "[|env \<in> list(A);  p \<in> formula;  arity(p) \<le> succ(length(env))|]
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   434
   ==> {x\<in>A. sats(A, p, Cons(x,env))} \<in> DPow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   435
by (simp add: DPow_def, blast) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   436
13291
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   437
text{*With this rule we can specify @{term p} later.*}
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   438
lemma DPowI2 [rule_format]:
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   439
  "[|\<forall>x\<in>A. P(x) <-> sats(A, p, Cons(x,env));
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   440
     env \<in> list(A);  p \<in> formula;  arity(p) \<le> succ(length(env))|]
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   441
   ==> {x\<in>A. P(x)} \<in> DPow(A)"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   442
by (simp add: DPow_def, blast) 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   443
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   444
lemma DPowD:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   445
  "X \<in> DPow(A) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   446
   ==> X <= A &
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   447
       (\<exists>env \<in> list(A). 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   448
        \<exists>p \<in> formula. arity(p) \<le> succ(length(env)) & 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   449
                      X = {x\<in>A. sats(A, p, Cons(x,env))})"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   450
by (simp add: DPow_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   451
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   452
lemmas DPow_imp_subset = DPowD [THEN conjunct1]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   453
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   454
(*Lemma 1.2*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   455
lemma "[| p \<in> formula; env \<in> list(A); arity(p) \<le> succ(length(env)) |] 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   456
       ==> {x\<in>A. sats(A, p, Cons(x,env))} \<in> DPow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   457
by (blast intro: DPowI)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   458
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   459
lemma DPow_subset_Pow: "DPow(A) <= Pow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   460
by (simp add: DPow_def, blast)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   461
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   462
lemma empty_in_DPow: "0 \<in> DPow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   463
apply (simp add: DPow_def)
13339
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13328
diff changeset
   464
apply (rule_tac x=Nil in bexI) 
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   465
 apply (rule_tac x="Neg(Equal(0,0))" in bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   466
  apply (auto simp add: Un_least_lt_iff) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   467
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   468
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   469
lemma Compl_in_DPow: "X \<in> DPow(A) ==> (A-X) \<in> DPow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   470
apply (simp add: DPow_def, clarify, auto) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   471
apply (rule bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   472
 apply (rule_tac x="Neg(p)" in bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   473
  apply auto 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   474
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   475
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   476
lemma Int_in_DPow: "[| X \<in> DPow(A); Y \<in> DPow(A) |] ==> X Int Y \<in> DPow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   477
apply (simp add: DPow_def, auto) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   478
apply (rename_tac envp p envq q) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   479
apply (rule_tac x="envp@envq" in bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   480
 apply (rule_tac x="And(p, iterates(incr_bv1,length(envp),q))" in bexI)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   481
  apply typecheck
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   482
apply (rule conjI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   483
(*finally check the arity!*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   484
 apply (simp add: arity_iterates_incr_bv1_eq length_app Un_least_lt_iff)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   485
 apply (force intro: add_le_self le_trans) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   486
apply (simp add: arity_sats1_iff formula_add_params1, blast) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   487
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   488
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   489
lemma Un_in_DPow: "[| X \<in> DPow(A); Y \<in> DPow(A) |] ==> X Un Y \<in> DPow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   490
apply (subgoal_tac "X Un Y = A - ((A-X) Int (A-Y))") 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   491
apply (simp add: Int_in_DPow Compl_in_DPow) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   492
apply (simp add: DPow_def, blast) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   493
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   494
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   495
lemma singleton_in_DPow: "x \<in> A ==> {x} \<in> DPow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   496
apply (simp add: DPow_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   497
apply (rule_tac x="Cons(x,Nil)" in bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   498
 apply (rule_tac x="Equal(0,1)" in bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   499
  apply typecheck
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   500
apply (force simp add: succ_Un_distrib [symmetric])  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   501
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   502
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   503
lemma cons_in_DPow: "[| a \<in> A; X \<in> DPow(A) |] ==> cons(a,X) \<in> DPow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   504
apply (rule cons_eq [THEN subst]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   505
apply (blast intro: singleton_in_DPow Un_in_DPow) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   506
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   507
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   508
(*Part of Lemma 1.3*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   509
lemma Fin_into_DPow: "X \<in> Fin(A) ==> X \<in> DPow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   510
apply (erule Fin.induct) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   511
 apply (rule empty_in_DPow) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   512
apply (blast intro: cons_in_DPow) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   513
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   514
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   515
(*DPow is not monotonic.  For example, let A be some non-constructible set
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   516
  of natural numbers, and let B be nat.  Then A<=B and obviously A : DPow(A)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   517
  but A ~: DPow(B).*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   518
lemma DPow_mono: "A : DPow(B) ==> DPow(A) <= DPow(B)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   519
apply (simp add: DPow_def, auto) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   520
(*must use the formula defining A in B to relativize the new formula...*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   521
oops
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   522
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   523
lemma DPow_0: "DPow(0) = {0}" 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   524
by (blast intro: empty_in_DPow dest: DPow_imp_subset)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   525
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   526
lemma Finite_Pow_subset_Pow: "Finite(A) ==> Pow(A) <= DPow(A)" 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   527
by (blast intro: Fin_into_DPow Finite_into_Fin Fin_subset)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   528
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   529
lemma Finite_DPow_eq_Pow: "Finite(A) ==> DPow(A) = Pow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   530
apply (rule equalityI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   531
apply (rule DPow_subset_Pow) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   532
apply (erule Finite_Pow_subset_Pow) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   533
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   534
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   535
(*This may be true but the proof looks difficult, requiring relativization 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   536
lemma DPow_insert: "DPow (cons(a,A)) = DPow(A) Un {cons(a,X) . X: DPow(A)}"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   537
apply (rule equalityI, safe)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   538
oops
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   539
*)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   540
13298
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   541
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   542
subsection{*Internalized formulas for basic concepts*}
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   543
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   544
subsubsection{*The subset relation*}
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   545
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   546
constdefs subset_fm :: "[i,i]=>i"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   547
    "subset_fm(x,y) == Forall(Implies(Member(0,succ(x)), Member(0,succ(y))))"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   548
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   549
lemma subset_type [TC]: "[| x \<in> nat; y \<in> nat |] ==> subset_fm(x,y) \<in> formula"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   550
by (simp add: subset_fm_def) 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   551
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   552
lemma arity_subset_fm [simp]:
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   553
     "[| x \<in> nat; y \<in> nat |] ==> arity(subset_fm(x,y)) = succ(x) \<union> succ(y)"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   554
by (simp add: subset_fm_def succ_Un_distrib [symmetric]) 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   555
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   556
lemma sats_subset_fm [simp]:
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   557
   "[|x < length(env); y \<in> nat; env \<in> list(A); Transset(A)|]
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   558
    ==> sats(A, subset_fm(x,y), env) <-> nth(x,env) \<subseteq> nth(y,env)"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   559
apply (frule lt_length_in_nat, assumption)  
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   560
apply (simp add: subset_fm_def Transset_def) 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   561
apply (blast intro: nth_type) 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   562
done
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   563
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   564
subsubsection{*Transitive sets*}
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   565
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   566
constdefs transset_fm :: "i=>i"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   567
   "transset_fm(x) == Forall(Implies(Member(0,succ(x)), subset_fm(0,succ(x))))"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   568
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   569
lemma transset_type [TC]: "x \<in> nat ==> transset_fm(x) \<in> formula"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   570
by (simp add: transset_fm_def) 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   571
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   572
lemma arity_transset_fm [simp]:
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   573
     "x \<in> nat ==> arity(transset_fm(x)) = succ(x)"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   574
by (simp add: transset_fm_def succ_Un_distrib [symmetric]) 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   575
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   576
lemma sats_transset_fm [simp]:
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   577
   "[|x < length(env); env \<in> list(A); Transset(A)|]
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   578
    ==> sats(A, transset_fm(x), env) <-> Transset(nth(x,env))"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   579
apply (frule lt_nat_in_nat, erule length_type) 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   580
apply (simp add: transset_fm_def Transset_def) 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   581
apply (blast intro: nth_type) 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   582
done
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   583
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   584
subsubsection{*Ordinals*}
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   585
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   586
constdefs ordinal_fm :: "i=>i"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   587
   "ordinal_fm(x) == 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   588
      And(transset_fm(x), Forall(Implies(Member(0,succ(x)), transset_fm(0))))"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   589
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   590
lemma ordinal_type [TC]: "x \<in> nat ==> ordinal_fm(x) \<in> formula"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   591
by (simp add: ordinal_fm_def) 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   592
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   593
lemma arity_ordinal_fm [simp]:
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   594
     "x \<in> nat ==> arity(ordinal_fm(x)) = succ(x)"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   595
by (simp add: ordinal_fm_def succ_Un_distrib [symmetric]) 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   596
13306
6eebcddee32b more internalized formulas and separation proofs
paulson
parents: 13298
diff changeset
   597
lemma sats_ordinal_fm:
13298
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   598
   "[|x < length(env); env \<in> list(A); Transset(A)|]
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   599
    ==> sats(A, ordinal_fm(x), env) <-> Ord(nth(x,env))"
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   600
apply (frule lt_nat_in_nat, erule length_type) 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   601
apply (simp add: ordinal_fm_def Ord_def Transset_def)
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   602
apply (blast intro: nth_type) 
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   603
done
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   604
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   605
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   606
subsection{* Constant Lset: Levels of the Constructible Universe *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   607
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   608
constdefs Lset :: "i=>i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   609
    "Lset(i) == transrec(i, %x f. \<Union>y\<in>x. DPow(f`y))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   610
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   611
text{*NOT SUITABLE FOR REWRITING -- RECURSIVE!*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   612
lemma Lset: "Lset(i) = (UN j:i. DPow(Lset(j)))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   613
by (subst Lset_def [THEN def_transrec], simp)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   614
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   615
lemma LsetI: "[|y\<in>x; A \<in> DPow(Lset(y))|] ==> A \<in> Lset(x)";
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   616
by (subst Lset, blast)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   617
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   618
lemma LsetD: "A \<in> Lset(x) ==> \<exists>y\<in>x. A \<in> DPow(Lset(y))";
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   619
apply (insert Lset [of x]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   620
apply (blast intro: elim: equalityE) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   621
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   622
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   623
subsubsection{* Transitivity *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   624
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   625
lemma elem_subset_in_DPow: "[|X \<in> A; X \<subseteq> A|] ==> X \<in> DPow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   626
apply (simp add: Transset_def DPow_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   627
apply (rule_tac x="[X]" in bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   628
 apply (rule_tac x="Member(0,1)" in bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   629
  apply (auto simp add: Un_least_lt_iff) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   630
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   631
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   632
lemma Transset_subset_DPow: "Transset(A) ==> A <= DPow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   633
apply clarify  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   634
apply (simp add: Transset_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   635
apply (blast intro: elem_subset_in_DPow) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   636
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   637
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   638
lemma Transset_DPow: "Transset(A) ==> Transset(DPow(A))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   639
apply (simp add: Transset_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   640
apply (blast intro: elem_subset_in_DPow dest: DPowD) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   641
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   642
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   643
text{*Kunen's VI, 1.6 (a)*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   644
lemma Transset_Lset: "Transset(Lset(i))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   645
apply (rule_tac a=i in eps_induct)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   646
apply (subst Lset)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   647
apply (blast intro!: Transset_Union_family Transset_Un Transset_DPow)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   648
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   649
13291
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   650
lemma mem_Lset_imp_subset_Lset: "a \<in> Lset(i) ==> a \<subseteq> Lset(i)"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   651
apply (insert Transset_Lset) 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   652
apply (simp add: Transset_def) 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   653
done
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   654
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   655
subsubsection{* Monotonicity *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   656
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   657
text{*Kunen's VI, 1.6 (b)*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   658
lemma Lset_mono [rule_format]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   659
     "ALL j. i<=j --> Lset(i) <= Lset(j)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   660
apply (rule_tac a=i in eps_induct)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   661
apply (rule impI [THEN allI])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   662
apply (subst Lset)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   663
apply (subst Lset, blast) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   664
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   665
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   666
text{*This version lets us remove the premise @{term "Ord(i)"} sometimes.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   667
lemma Lset_mono_mem [rule_format]:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   668
     "ALL j. i:j --> Lset(i) <= Lset(j)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   669
apply (rule_tac a=i in eps_induct)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   670
apply (rule impI [THEN allI])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   671
apply (subst Lset, auto) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   672
apply (rule rev_bexI, assumption)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   673
apply (blast intro: elem_subset_in_DPow dest: LsetD DPowD) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   674
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   675
13291
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   676
text{*Useful with Reflection to bump up the ordinal*}
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   677
lemma subset_Lset_ltD: "[|A \<subseteq> Lset(i); i < j|] ==> A \<subseteq> Lset(j)"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   678
by (blast dest: ltD [THEN Lset_mono_mem]) 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   679
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   680
subsubsection{* 0, successor and limit equations fof Lset *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   681
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   682
lemma Lset_0 [simp]: "Lset(0) = 0"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   683
by (subst Lset, blast)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   684
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   685
lemma Lset_succ_subset1: "DPow(Lset(i)) <= Lset(succ(i))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   686
by (subst Lset, rule succI1 [THEN RepFunI, THEN Union_upper])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   687
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   688
lemma Lset_succ_subset2: "Lset(succ(i)) <= DPow(Lset(i))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   689
apply (subst Lset, rule UN_least)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   690
apply (erule succE) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   691
 apply blast 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   692
apply clarify
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   693
apply (rule elem_subset_in_DPow)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   694
 apply (subst Lset)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   695
 apply blast 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   696
apply (blast intro: dest: DPowD Lset_mono_mem) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   697
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   698
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   699
lemma Lset_succ: "Lset(succ(i)) = DPow(Lset(i))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   700
by (intro equalityI Lset_succ_subset1 Lset_succ_subset2) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   701
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   702
lemma Lset_Union [simp]: "Lset(\<Union>(X)) = (\<Union>y\<in>X. Lset(y))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   703
apply (subst Lset)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   704
apply (rule equalityI)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   705
 txt{*first inclusion*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   706
 apply (rule UN_least)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   707
 apply (erule UnionE)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   708
 apply (rule subset_trans)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   709
  apply (erule_tac [2] UN_upper, subst Lset, erule UN_upper)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   710
txt{*opposite inclusion*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   711
apply (rule UN_least)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   712
apply (subst Lset, blast)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   713
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   714
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   715
subsubsection{* Lset applied to Limit ordinals *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   716
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   717
lemma Limit_Lset_eq:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   718
    "Limit(i) ==> Lset(i) = (\<Union>y\<in>i. Lset(y))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   719
by (simp add: Lset_Union [symmetric] Limit_Union_eq)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   720
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   721
lemma lt_LsetI: "[| a: Lset(j);  j<i |] ==> a : Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   722
by (blast dest: Lset_mono [OF le_imp_subset [OF leI]])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   723
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   724
lemma Limit_LsetE:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   725
    "[| a: Lset(i);  ~R ==> Limit(i);
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   726
        !!x. [| x<i;  a: Lset(x) |] ==> R
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   727
     |] ==> R"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   728
apply (rule classical)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   729
apply (rule Limit_Lset_eq [THEN equalityD1, THEN subsetD, THEN UN_E])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   730
  prefer 2 apply assumption
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   731
 apply blast 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   732
apply (blast intro: ltI  Limit_is_Ord)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   733
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   734
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   735
subsubsection{* Basic closure properties *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   736
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   737
lemma zero_in_Lset: "y:x ==> 0 : Lset(x)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   738
by (subst Lset, blast intro: empty_in_DPow)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   739
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   740
lemma notin_Lset: "x \<notin> Lset(x)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   741
apply (rule_tac a=x in eps_induct)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   742
apply (subst Lset)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   743
apply (blast dest: DPowD)  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   744
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   745
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   746
13298
b4f370679c65 Constructible: some separation axioms
paulson
parents: 13291
diff changeset
   747
subsection{*Constructible Ordinals: Kunen's VI, 1.9 (b)*}
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   748
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   749
text{*The subset consisting of the ordinals is definable.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   750
lemma Ords_in_DPow: "Transset(A) ==> {x \<in> A. Ord(x)} \<in> DPow(A)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   751
apply (simp add: DPow_def Collect_subset) 
13339
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13328
diff changeset
   752
apply (rule_tac x=Nil in bexI) 
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   753
 apply (rule_tac x="ordinal_fm(0)" in bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   754
apply (simp_all add: sats_ordinal_fm)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   755
done 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   756
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   757
lemma Ords_of_Lset_eq: "Ord(i) ==> {x\<in>Lset(i). Ord(x)} = i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   758
apply (erule trans_induct3)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   759
  apply (simp_all add: Lset_succ Limit_Lset_eq Limit_Union_eq)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   760
txt{*The successor case remains.*} 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   761
apply (rule equalityI)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   762
txt{*First inclusion*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   763
 apply clarify  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   764
 apply (erule Ord_linear_lt, assumption) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   765
   apply (blast dest: DPow_imp_subset ltD notE [OF notin_Lset]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   766
  apply blast 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   767
 apply (blast dest: ltD)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   768
txt{*Opposite inclusion, @{term "succ(x) \<subseteq> DPow(Lset(x)) \<inter> ON"}*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   769
apply auto
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   770
txt{*Key case: *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   771
  apply (erule subst, rule Ords_in_DPow [OF Transset_Lset]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   772
 apply (blast intro: elem_subset_in_DPow dest: OrdmemD elim: equalityE) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   773
apply (blast intro: Ord_in_Ord) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   774
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   775
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   776
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   777
lemma Ord_subset_Lset: "Ord(i) ==> i \<subseteq> Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   778
by (subst Ords_of_Lset_eq [symmetric], assumption, fast)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   779
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   780
lemma Ord_in_Lset: "Ord(i) ==> i \<in> Lset(succ(i))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   781
apply (simp add: Lset_succ)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   782
apply (subst Ords_of_Lset_eq [symmetric], assumption, 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   783
       rule Ords_in_DPow [OF Transset_Lset]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   784
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   785
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   786
subsubsection{* Unions *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   787
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   788
lemma Union_in_Lset:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   789
     "X \<in> Lset(j) ==> Union(X) \<in> Lset(succ(j))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   790
apply (insert Transset_Lset)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   791
apply (rule LsetI [OF succI1])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   792
apply (simp add: Transset_def DPow_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   793
apply (intro conjI, blast)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   794
txt{*Now to create the formula @{term "\<exists>y. y \<in> X \<and> x \<in> y"} *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   795
apply (rule_tac x="Cons(X,Nil)" in bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   796
 apply (rule_tac x="Exists(And(Member(0,2), Member(1,0)))" in bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   797
  apply typecheck
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   798
apply (simp add: succ_Un_distrib [symmetric], blast) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   799
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   800
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   801
lemma Union_in_LLimit:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   802
     "[| X: Lset(i);  Limit(i) |] ==> Union(X) : Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   803
apply (rule Limit_LsetE, assumption+)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   804
apply (blast intro: Limit_has_succ lt_LsetI Union_in_Lset)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   805
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   806
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   807
subsubsection{* Finite sets and ordered pairs *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   808
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   809
lemma singleton_in_Lset: "a: Lset(i) ==> {a} : Lset(succ(i))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   810
by (simp add: Lset_succ singleton_in_DPow) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   811
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   812
lemma doubleton_in_Lset:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   813
     "[| a: Lset(i);  b: Lset(i) |] ==> {a,b} : Lset(succ(i))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   814
by (simp add: Lset_succ empty_in_DPow cons_in_DPow) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   815
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   816
lemma Pair_in_Lset:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   817
    "[| a: Lset(i);  b: Lset(i); Ord(i) |] ==> <a,b> : Lset(succ(succ(i)))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   818
apply (unfold Pair_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   819
apply (blast intro: doubleton_in_Lset) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   820
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   821
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   822
lemmas zero_in_LLimit = Limit_has_0 [THEN ltD, THEN zero_in_Lset, standard]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   823
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   824
lemma singleton_in_LLimit:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   825
    "[| a: Lset(i);  Limit(i) |] ==> {a} : Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   826
apply (erule Limit_LsetE, assumption)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   827
apply (erule singleton_in_Lset [THEN lt_LsetI])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   828
apply (blast intro: Limit_has_succ) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   829
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   830
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   831
lemmas Lset_UnI1 = Un_upper1 [THEN Lset_mono [THEN subsetD], standard]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   832
lemmas Lset_UnI2 = Un_upper2 [THEN Lset_mono [THEN subsetD], standard]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   833
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   834
text{*Hard work is finding a single j:i such that {a,b}<=Lset(j)*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   835
lemma doubleton_in_LLimit:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   836
    "[| a: Lset(i);  b: Lset(i);  Limit(i) |] ==> {a,b} : Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   837
apply (erule Limit_LsetE, assumption)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   838
apply (erule Limit_LsetE, assumption)
13269
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   839
apply (blast intro: lt_LsetI [OF doubleton_in_Lset]
3ba9be497c33 Tidying and introduction of various new theorems
paulson
parents: 13245
diff changeset
   840
                    Lset_UnI1 Lset_UnI2 Limit_has_succ Un_least_lt)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   841
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   842
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   843
lemma Pair_in_LLimit:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   844
    "[| a: Lset(i);  b: Lset(i);  Limit(i) |] ==> <a,b> : Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   845
txt{*Infer that a, b occur at ordinals x,xa < i.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   846
apply (erule Limit_LsetE, assumption)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   847
apply (erule Limit_LsetE, assumption)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   848
txt{*Infer that succ(succ(x Un xa)) < i *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   849
apply (blast intro: lt_Ord lt_LsetI [OF Pair_in_Lset]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   850
                    Lset_UnI1 Lset_UnI2 Limit_has_succ Un_least_lt)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   851
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   852
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   853
lemma product_LLimit: "Limit(i) ==> Lset(i) * Lset(i) <= Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   854
by (blast intro: Pair_in_LLimit)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   855
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   856
lemmas Sigma_subset_LLimit = subset_trans [OF Sigma_mono product_LLimit]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   857
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   858
lemma nat_subset_LLimit: "Limit(i) ==> nat \<subseteq> Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   859
by (blast dest: Ord_subset_Lset nat_le_Limit le_imp_subset Limit_is_Ord)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   860
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   861
lemma nat_into_LLimit: "[| n: nat;  Limit(i) |] ==> n : Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   862
by (blast intro: nat_subset_LLimit [THEN subsetD])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   863
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   864
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   865
subsubsection{* Closure under disjoint union *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   866
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   867
lemmas zero_in_LLimit = Limit_has_0 [THEN ltD, THEN zero_in_Lset, standard]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   868
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   869
lemma one_in_LLimit: "Limit(i) ==> 1 : Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   870
by (blast intro: nat_into_LLimit)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   871
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   872
lemma Inl_in_LLimit:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   873
    "[| a: Lset(i); Limit(i) |] ==> Inl(a) : Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   874
apply (unfold Inl_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   875
apply (blast intro: zero_in_LLimit Pair_in_LLimit)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   876
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   877
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   878
lemma Inr_in_LLimit:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   879
    "[| b: Lset(i); Limit(i) |] ==> Inr(b) : Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   880
apply (unfold Inr_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   881
apply (blast intro: one_in_LLimit Pair_in_LLimit)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   882
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   883
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   884
lemma sum_LLimit: "Limit(i) ==> Lset(i) + Lset(i) <= Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   885
by (blast intro!: Inl_in_LLimit Inr_in_LLimit)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   886
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   887
lemmas sum_subset_LLimit = subset_trans [OF sum_mono sum_LLimit]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   888
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   889
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   890
text{*The constructible universe and its rank function*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   891
constdefs
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   892
  L :: "i=>o" --{*Kunen's definition VI, 1.5, page 167*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   893
    "L(x) == \<exists>i. Ord(i) & x \<in> Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   894
  
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   895
  lrank :: "i=>i" --{*Kunen's definition VI, 1.7*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   896
    "lrank(x) == \<mu>i. x \<in> Lset(succ(i))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   897
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   898
lemma L_I: "[|x \<in> Lset(i); Ord(i)|] ==> L(x)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   899
by (simp add: L_def, blast)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   900
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   901
lemma L_D: "L(x) ==> \<exists>i. Ord(i) & x \<in> Lset(i)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   902
by (simp add: L_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   903
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   904
lemma Ord_lrank [simp]: "Ord(lrank(a))"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   905
by (simp add: lrank_def)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   906
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   907
lemma Lset_lrank_lt [rule_format]: "Ord(i) ==> x \<in> Lset(i) --> lrank(x) < i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   908
apply (erule trans_induct3)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   909
  apply simp   
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   910
 apply (simp only: lrank_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   911
 apply (blast intro: Least_le) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   912
apply (simp_all add: Limit_Lset_eq) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   913
apply (blast intro: ltI Limit_is_Ord lt_trans) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   914
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   915
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   916
text{*Kunen's VI, 1.8, and the proof is much less trivial than the text
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   917
would suggest.  For a start it need the previous lemma, proved by induction.*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   918
lemma Lset_iff_lrank_lt: "Ord(i) ==> x \<in> Lset(i) <-> L(x) & lrank(x) < i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   919
apply (simp add: L_def, auto) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   920
 apply (blast intro: Lset_lrank_lt) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   921
 apply (unfold lrank_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   922
apply (drule succI1 [THEN Lset_mono_mem, THEN subsetD]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   923
apply (drule_tac P="\<lambda>i. x \<in> Lset(succ(i))" in LeastI, assumption) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   924
apply (blast intro!: le_imp_subset Lset_mono [THEN subsetD]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   925
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   926
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   927
lemma Lset_succ_lrank_iff [simp]: "x \<in> Lset(succ(lrank(x))) <-> L(x)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   928
by (simp add: Lset_iff_lrank_lt)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   929
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   930
text{*Kunen's VI, 1.9 (a)*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   931
lemma lrank_of_Ord: "Ord(i) ==> lrank(i) = i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   932
apply (unfold lrank_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   933
apply (rule Least_equality) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   934
  apply (erule Ord_in_Lset) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   935
 apply assumption
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   936
apply (insert notin_Lset [of i]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   937
apply (blast intro!: le_imp_subset Lset_mono [THEN subsetD]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   938
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   939
13245
714f7a423a15 development and tweaks
paulson
parents: 13223
diff changeset
   940
714f7a423a15 development and tweaks
paulson
parents: 13223
diff changeset
   941
lemma Ord_in_L: "Ord(i) ==> L(i)"
714f7a423a15 development and tweaks
paulson
parents: 13223
diff changeset
   942
by (blast intro: Ord_in_Lset L_I)
714f7a423a15 development and tweaks
paulson
parents: 13223
diff changeset
   943
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   944
text{*This is lrank(lrank(a)) = lrank(a) *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   945
declare Ord_lrank [THEN lrank_of_Ord, simp]
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   946
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   947
text{*Kunen's VI, 1.10 *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   948
lemma Lset_in_Lset_succ: "Lset(i) \<in> Lset(succ(i))";
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   949
apply (simp add: Lset_succ DPow_def) 
13339
0f89104dd377 Fixed quantified variable name preservation for ball and bex (bounded quants)
paulson
parents: 13328
diff changeset
   950
apply (rule_tac x=Nil in bexI) 
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   951
 apply (rule_tac x="Equal(0,0)" in bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   952
apply auto 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   953
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   954
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   955
lemma lrank_Lset: "Ord(i) ==> lrank(Lset(i)) = i"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   956
apply (unfold lrank_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   957
apply (rule Least_equality) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   958
  apply (rule Lset_in_Lset_succ) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   959
 apply assumption
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   960
apply clarify 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   961
apply (subgoal_tac "Lset(succ(ia)) <= Lset(i)")
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   962
 apply (blast dest: mem_irrefl) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   963
apply (blast intro!: le_imp_subset Lset_mono) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   964
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   965
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   966
text{*Kunen's VI, 1.11 *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   967
lemma Lset_subset_Vset: "Ord(i) ==> Lset(i) <= Vset(i)";
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   968
apply (erule trans_induct)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   969
apply (subst Lset) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   970
apply (subst Vset) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   971
apply (rule UN_mono [OF subset_refl]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   972
apply (rule subset_trans [OF DPow_subset_Pow]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   973
apply (rule Pow_mono, blast) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   974
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   975
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   976
text{*Kunen's VI, 1.12 *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   977
lemma Lset_subset_Vset: "i \<in> nat ==> Lset(i) = Vset(i)";
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   978
apply (erule nat_induct)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   979
 apply (simp add: Vfrom_0) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   980
apply (simp add: Lset_succ Vset_succ Finite_Vset Finite_DPow_eq_Pow) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   981
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   982
13291
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   983
text{*Every set of constructible sets is included in some @{term Lset}*} 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   984
lemma subset_Lset:
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   985
     "(\<forall>x\<in>A. L(x)) ==> \<exists>i. Ord(i) & A \<subseteq> Lset(i)"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   986
by (rule_tac x = "\<Union>x\<in>A. succ(lrank(x))" in exI, force)
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   987
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   988
lemma subset_LsetE:
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   989
     "[|\<forall>x\<in>A. L(x);
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   990
        !!i. [|Ord(i); A \<subseteq> Lset(i)|] ==> P|]
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   991
      ==> P"
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   992
by (blast dest: subset_Lset) 
a73ab154f75c towards proving separation for L
paulson
parents: 13269
diff changeset
   993
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   994
subsection{*For L to satisfy the ZF axioms*}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   995
13245
714f7a423a15 development and tweaks
paulson
parents: 13223
diff changeset
   996
theorem Union_in_L: "L(X) ==> L(Union(X))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   997
apply (simp add: L_def, clarify) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   998
apply (drule Ord_imp_greater_Limit) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
   999
apply (blast intro: lt_LsetI Union_in_LLimit Limit_is_Ord) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1000
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1001
13245
714f7a423a15 development and tweaks
paulson
parents: 13223
diff changeset
  1002
theorem doubleton_in_L: "[| L(a); L(b) |] ==> L({a, b})"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1003
apply (simp add: L_def, clarify) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1004
apply (drule Ord2_imp_greater_Limit, assumption) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1005
apply (blast intro: lt_LsetI doubleton_in_LLimit Limit_is_Ord) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1006
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1007
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1008
subsubsection{*For L to satisfy Powerset *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1009
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1010
lemma LPow_env_typing:
13511
e4b129eaa9c6 new proof needed now
paulson
parents: 13505
diff changeset
  1011
    "[| y : Lset(i); Ord(i); y \<subseteq> X |] 
e4b129eaa9c6 new proof needed now
paulson
parents: 13505
diff changeset
  1012
     ==> \<exists>z \<in> Pow(X). y \<in> Lset(succ(lrank(z)))"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1013
by (auto intro: L_I iff: Lset_succ_lrank_iff) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1014
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1015
lemma LPow_in_Lset:
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1016
     "[|X \<in> Lset(i); Ord(i)|] ==> \<exists>j. Ord(j) & {y \<in> Pow(X). L(y)} \<in> Lset(j)"
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1017
apply (rule_tac x="succ(\<Union>y \<in> Pow(X). succ(lrank(y)))" in exI)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1018
apply simp 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1019
apply (rule LsetI [OF succI1])
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1020
apply (simp add: DPow_def) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1021
apply (intro conjI, clarify) 
13511
e4b129eaa9c6 new proof needed now
paulson
parents: 13505
diff changeset
  1022
 apply (rule_tac a=x in UN_I, simp+)  
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1023
txt{*Now to create the formula @{term "y \<subseteq> X"} *}
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1024
apply (rule_tac x="Cons(X,Nil)" in bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1025
 apply (rule_tac x="subset_fm(0,1)" in bexI) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1026
  apply typecheck
13511
e4b129eaa9c6 new proof needed now
paulson
parents: 13505
diff changeset
  1027
 apply (rule conjI) 
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1028
apply (simp add: succ_Un_distrib [symmetric]) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1029
apply (rule equality_iffI) 
13511
e4b129eaa9c6 new proof needed now
paulson
parents: 13505
diff changeset
  1030
apply (simp add: Transset_UN [OF Transset_Lset] LPow_env_typing)
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1031
apply (auto intro: L_I iff: Lset_succ_lrank_iff) 
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1032
done
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1033
13245
714f7a423a15 development and tweaks
paulson
parents: 13223
diff changeset
  1034
theorem LPow_in_L: "L(X) ==> L({y \<in> Pow(X). L(y)})"
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1035
by (blast intro: L_I dest: L_D LPow_in_Lset)
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1036
13385
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1037
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1038
subsection{*Eliminating @{term arity} from the Definition of @{term Lset}*}
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1039
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1040
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1041
lemma nth_zero_eq_0: "n \<in> nat ==> nth(n,[0]) = 0"
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1042
by (induct_tac n, auto)
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1043
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1044
lemma sats_app_0_iff [rule_format]:
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1045
  "[| p \<in> formula; 0 \<in> A |]
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1046
   ==> \<forall>env \<in> list(A). sats(A,p, env@[0]) <-> sats(A,p,env)"
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1047
apply (induct_tac p)
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1048
apply (simp_all del: app_Cons add: app_Cons [symmetric]
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1049
		add: nth_zero_eq_0 nth_append not_lt_iff_le nth_eq_0)
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1050
done
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1051
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1052
lemma sats_app_zeroes_iff:
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1053
  "[| p \<in> formula; 0 \<in> A; env \<in> list(A); n \<in> nat |]
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1054
   ==> sats(A,p,env @ repeat(0,n)) <-> sats(A,p,env)"
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1055
apply (induct_tac n, simp) 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1056
apply (simp del: repeat.simps
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1057
            add: repeat_succ_app sats_app_0_iff app_assoc [symmetric]) 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1058
done
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1059
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1060
lemma exists_bigger_env:
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1061
  "[| p \<in> formula; 0 \<in> A; env \<in> list(A) |]
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1062
   ==> \<exists>env' \<in> list(A). arity(p) \<le> succ(length(env')) & 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1063
              (\<forall>a\<in>A. sats(A,p,Cons(a,env')) <-> sats(A,p,Cons(a,env)))"
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1064
apply (rule_tac x="env @ repeat(0,arity(p))" in bexI) 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1065
apply (simp del: app_Cons add: app_Cons [symmetric]
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1066
	    add: length_repeat sats_app_zeroes_iff, typecheck)
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1067
done
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1068
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1069
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1070
text{*A simpler version of @{term DPow}: no arity check!*}
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1071
constdefs DPow' :: "i => i"
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1072
  "DPow'(A) == {X \<in> Pow(A). 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1073
                \<exists>env \<in> list(A). \<exists>p \<in> formula. 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1074
                    X = {x\<in>A. sats(A, p, Cons(x,env))}}"
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1075
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1076
lemma DPow_subset_DPow': "DPow(A) <= DPow'(A)";
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1077
by (simp add: DPow_def DPow'_def, blast)
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1078
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1079
lemma DPow'_0: "DPow'(0) = {0}"
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1080
by (auto simp add: DPow'_def)
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1081
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1082
lemma DPow'_subset_DPow: "0 \<in> A ==> DPow'(A) \<subseteq> DPow(A)"
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1083
apply (auto simp add: DPow'_def DPow_def) 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1084
apply (frule exists_bigger_env, assumption+, force)  
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1085
done
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1086
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1087
lemma DPow_eq_DPow': "Transset(A) ==> DPow(A) = DPow'(A)"
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1088
apply (drule Transset_0_disj) 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1089
apply (erule disjE) 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1090
 apply (simp add: DPow'_0 DPow_0) 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1091
apply (rule equalityI)
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1092
 apply (rule DPow_subset_DPow') 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1093
apply (erule DPow'_subset_DPow) 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1094
done
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1095
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1096
text{*And thus we can relativize @{term Lset} without bothering with
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1097
      @{term arity} and @{term length}*}
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1098
lemma Lset_eq_transrec_DPow': "Lset(i) = transrec(i, %x f. \<Union>y\<in>x. DPow'(f`y))"
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1099
apply (rule_tac a=i in eps_induct)
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1100
apply (subst Lset)
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1101
apply (subst transrec)
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1102
apply (simp only: DPow_eq_DPow' [OF Transset_Lset], simp) 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1103
done
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1104
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1105
text{*With this rule we can specify @{term p} later and don't worry about
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1106
      arities at all!*}
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1107
lemma DPow_LsetI [rule_format]:
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1108
  "[|\<forall>x\<in>Lset(i). P(x) <-> sats(Lset(i), p, Cons(x,env));
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1109
     env \<in> list(Lset(i));  p \<in> formula|]
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1110
   ==> {x\<in>Lset(i). P(x)} \<in> DPow(Lset(i))"
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1111
by (simp add: DPow_eq_DPow' [OF Transset_Lset] DPow'_def, blast) 
31df66ca0780 Expressing Lset and L without using length and arity; simplifies Separation
paulson
parents: 13339
diff changeset
  1112
13223
45be08fbdcff new theory of inner models
paulson
parents:
diff changeset
  1113
end