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