| author | blanchet | 
| Sat, 08 Sep 2012 21:30:31 +0200 | |
| changeset 49222 | cbe8c859817c | 
| parent 47398 | 07bcf80391d0 | 
| child 49660 | de49d9b4d7bc | 
| permissions | -rw-r--r-- | 
| 32139 | 1 | (* Author: Tobias Nipkow, Lawrence C Paulson and Markus Wenzel *) | 
| 923 | 2 | |
| 11979 | 3 | header {* Set theory for higher-order logic *}
 | 
| 4 | ||
| 15131 | 5 | theory Set | 
| 30304 
d8e4cd2ac2a1
set operations Int, Un, INTER, UNION, Inter, Union, empty, UNIV are now proper qualified constants with authentic syntax
 haftmann parents: 
29901diff
changeset | 6 | imports Lattices | 
| 15131 | 7 | begin | 
| 11979 | 8 | |
| 32081 | 9 | subsection {* Sets as predicates *}
 | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 10 | |
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 11 | typedecl 'a set | 
| 3820 | 12 | |
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 13 | axiomatization Collect :: "('a \<Rightarrow> bool) \<Rightarrow> 'a set" -- "comprehension"
 | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 14 | and member :: "'a \<Rightarrow> 'a set \<Rightarrow> bool" -- "membership" | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 15 | where | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 16 | mem_Collect_eq [iff, code_unfold]: "member a (Collect P) = P a" | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 17 | and Collect_mem_eq [simp]: "Collect (\<lambda>x. member x A) = A" | 
| 19656 
09be06943252
tuned concrete syntax -- abbreviation/const_syntax;
 wenzelm parents: 
19637diff
changeset | 18 | |
| 21210 | 19 | notation | 
| 37677 | 20 |   member  ("op :") and
 | 
| 21 |   member  ("(_/ : _)" [50, 51] 50)
 | |
| 11979 | 22 | |
| 37677 | 23 | abbreviation not_member where | 
| 24 | "not_member x A \<equiv> ~ (x : A)" -- "non-membership" | |
| 19656 
09be06943252
tuned concrete syntax -- abbreviation/const_syntax;
 wenzelm parents: 
19637diff
changeset | 25 | |
| 21210 | 26 | notation | 
| 37677 | 27 |   not_member  ("op ~:") and
 | 
| 28 |   not_member  ("(_/ ~: _)" [50, 51] 50)
 | |
| 19656 
09be06943252
tuned concrete syntax -- abbreviation/const_syntax;
 wenzelm parents: 
19637diff
changeset | 29 | |
| 21210 | 30 | notation (xsymbols) | 
| 37677 | 31 |   member      ("op \<in>") and
 | 
| 32 |   member      ("(_/ \<in> _)" [50, 51] 50) and
 | |
| 33 |   not_member  ("op \<notin>") and
 | |
| 34 |   not_member  ("(_/ \<notin> _)" [50, 51] 50)
 | |
| 19656 
09be06943252
tuned concrete syntax -- abbreviation/const_syntax;
 wenzelm parents: 
19637diff
changeset | 35 | |
| 21210 | 36 | notation (HTML output) | 
| 37677 | 37 |   member      ("op \<in>") and
 | 
| 38 |   member      ("(_/ \<in> _)" [50, 51] 50) and
 | |
| 39 |   not_member  ("op \<notin>") and
 | |
| 40 |   not_member  ("(_/ \<notin> _)" [50, 51] 50)
 | |
| 19656 
09be06943252
tuned concrete syntax -- abbreviation/const_syntax;
 wenzelm parents: 
19637diff
changeset | 41 | |
| 41107 | 42 | |
| 32081 | 43 | text {* Set comprehensions *}
 | 
| 44 | ||
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 45 | syntax | 
| 35115 | 46 |   "_Coll" :: "pttrn => bool => 'a set"    ("(1{_./ _})")
 | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 47 | translations | 
| 35115 | 48 |   "{x. P}" == "CONST Collect (%x. P)"
 | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 49 | |
| 32081 | 50 | syntax | 
| 35115 | 51 |   "_Collect" :: "idt => 'a set => bool => 'a set"    ("(1{_ :/ _./ _})")
 | 
| 32081 | 52 | syntax (xsymbols) | 
| 35115 | 53 |   "_Collect" :: "idt => 'a set => bool => 'a set"    ("(1{_ \<in>/ _./ _})")
 | 
| 32081 | 54 | translations | 
| 35115 | 55 |   "{x:A. P}" => "{x. x:A & P}"
 | 
| 32081 | 56 | |
| 41107 | 57 | lemma CollectI: "P a \<Longrightarrow> a \<in> {x. P x}"
 | 
| 32081 | 58 | by simp | 
| 59 | ||
| 41107 | 60 | lemma CollectD: "a \<in> {x. P x} \<Longrightarrow> P a"
 | 
| 32081 | 61 | by simp | 
| 62 | ||
| 41107 | 63 | lemma Collect_cong: "(\<And>x. P x = Q x) ==> {x. P x} = {x. Q x}"
 | 
| 32081 | 64 | by simp | 
| 65 | ||
| 32117 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 66 | text {*
 | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 67 | Simproc for pulling @{text "x=t"} in @{text "{x. \<dots> & x=t & \<dots>}"}
 | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 68 | to the front (and similarly for @{text "t=x"}):
 | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 69 | *} | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 70 | |
| 42455 | 71 | simproc_setup defined_Collect ("{x. P x & Q x}") = {*
 | 
| 42459 | 72 | fn _ => | 
| 73 | Quantifier1.rearrange_Collect | |
| 74 |      (rtac @{thm Collect_cong} 1 THEN
 | |
| 42455 | 75 |       rtac @{thm iffI} 1 THEN
 | 
| 42459 | 76 | ALLGOALS | 
| 77 |         (EVERY' [REPEAT_DETERM o etac @{thm conjE}, DEPTH_SOLVE_1 o ares_tac @{thms conjI}]))
 | |
| 32117 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 78 | *} | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 79 | |
| 32081 | 80 | lemmas CollectE = CollectD [elim_format] | 
| 81 | ||
| 41107 | 82 | lemma set_eqI: | 
| 83 | assumes "\<And>x. x \<in> A \<longleftrightarrow> x \<in> B" | |
| 84 | shows "A = B" | |
| 85 | proof - | |
| 86 |   from assms have "{x. x \<in> A} = {x. x \<in> B}" by simp
 | |
| 87 | then show ?thesis by simp | |
| 88 | qed | |
| 89 | ||
| 90 | lemma set_eq_iff [no_atp]: | |
| 91 | "A = B \<longleftrightarrow> (\<forall>x. x \<in> A \<longleftrightarrow> x \<in> B)" | |
| 92 | by (auto intro:set_eqI) | |
| 93 | ||
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 94 | text {* Lifting of predicate class instances *}
 | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 95 | |
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 96 | instantiation set :: (type) boolean_algebra | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 97 | begin | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 98 | |
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 99 | definition less_eq_set where | 
| 46853 | 100 | "A \<le> B \<longleftrightarrow> (\<lambda>x. member x A) \<le> (\<lambda>x. member x B)" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 101 | |
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 102 | definition less_set where | 
| 46853 | 103 | "A < B \<longleftrightarrow> (\<lambda>x. member x A) < (\<lambda>x. member x B)" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 104 | |
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 105 | definition inf_set where | 
| 46853 | 106 | "A \<sqinter> B = Collect ((\<lambda>x. member x A) \<sqinter> (\<lambda>x. member x B))" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 107 | |
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 108 | definition sup_set where | 
| 46853 | 109 | "A \<squnion> B = Collect ((\<lambda>x. member x A) \<squnion> (\<lambda>x. member x B))" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 110 | |
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 111 | definition bot_set where | 
| 46853 | 112 | "\<bottom> = Collect \<bottom>" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 113 | |
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 114 | definition top_set where | 
| 46853 | 115 | "\<top> = Collect \<top>" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 116 | |
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 117 | definition uminus_set where | 
| 46853 | 118 | "- A = Collect (- (\<lambda>x. member x A))" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 119 | |
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 120 | definition minus_set where | 
| 46853 | 121 | "A - B = Collect ((\<lambda>x. member x A) - (\<lambda>x. member x B))" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 122 | |
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 123 | instance proof | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 124 | qed (simp_all add: less_eq_set_def less_set_def inf_set_def sup_set_def | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 125 | bot_set_def top_set_def uminus_set_def minus_set_def | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 126 | less_le_not_le inf_compl_bot sup_compl_top sup_inf_distrib1 diff_eq | 
| 46882 | 127 | set_eqI fun_eq_iff | 
| 128 | del: inf_apply sup_apply bot_apply top_apply minus_apply uminus_apply) | |
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 129 | |
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 130 | end | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 131 | |
| 32081 | 132 | text {* Set enumerations *}
 | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 133 | |
| 32264 
0be31453f698
Set.UNIV and Set.empty are mere abbreviations for top and bot
 haftmann parents: 
32139diff
changeset | 134 | abbreviation empty :: "'a set" ("{}") where
 | 
| 
0be31453f698
Set.UNIV and Set.empty are mere abbreviations for top and bot
 haftmann parents: 
32139diff
changeset | 135 |   "{} \<equiv> bot"
 | 
| 31456 | 136 | |
| 137 | definition insert :: "'a \<Rightarrow> 'a set \<Rightarrow> 'a set" where | |
| 32081 | 138 |   insert_compr: "insert a B = {x. x = a \<or> x \<in> B}"
 | 
| 31456 | 139 | |
| 140 | syntax | |
| 35115 | 141 |   "_Finset" :: "args => 'a set"    ("{(_)}")
 | 
| 31456 | 142 | translations | 
| 35115 | 143 |   "{x, xs}" == "CONST insert x {xs}"
 | 
| 144 |   "{x}" == "CONST insert x {}"
 | |
| 31456 | 145 | |
| 32081 | 146 | |
| 147 | subsection {* Subsets and bounded quantifiers *}
 | |
| 148 | ||
| 149 | abbreviation | |
| 150 | subset :: "'a set \<Rightarrow> 'a set \<Rightarrow> bool" where | |
| 151 | "subset \<equiv> less" | |
| 152 | ||
| 153 | abbreviation | |
| 154 | subset_eq :: "'a set \<Rightarrow> 'a set \<Rightarrow> bool" where | |
| 155 | "subset_eq \<equiv> less_eq" | |
| 156 | ||
| 157 | notation (output) | |
| 158 |   subset  ("op <") and
 | |
| 159 |   subset  ("(_/ < _)" [50, 51] 50) and
 | |
| 160 |   subset_eq  ("op <=") and
 | |
| 161 |   subset_eq  ("(_/ <= _)" [50, 51] 50)
 | |
| 162 | ||
| 163 | notation (xsymbols) | |
| 164 |   subset  ("op \<subset>") and
 | |
| 165 |   subset  ("(_/ \<subset> _)" [50, 51] 50) and
 | |
| 166 |   subset_eq  ("op \<subseteq>") and
 | |
| 167 |   subset_eq  ("(_/ \<subseteq> _)" [50, 51] 50)
 | |
| 168 | ||
| 169 | notation (HTML output) | |
| 170 |   subset  ("op \<subset>") and
 | |
| 171 |   subset  ("(_/ \<subset> _)" [50, 51] 50) and
 | |
| 172 |   subset_eq  ("op \<subseteq>") and
 | |
| 173 |   subset_eq  ("(_/ \<subseteq> _)" [50, 51] 50)
 | |
| 174 | ||
| 175 | abbreviation (input) | |
| 176 | supset :: "'a set \<Rightarrow> 'a set \<Rightarrow> bool" where | |
| 177 | "supset \<equiv> greater" | |
| 178 | ||
| 179 | abbreviation (input) | |
| 180 | supset_eq :: "'a set \<Rightarrow> 'a set \<Rightarrow> bool" where | |
| 181 | "supset_eq \<equiv> greater_eq" | |
| 182 | ||
| 183 | notation (xsymbols) | |
| 184 |   supset  ("op \<supset>") and
 | |
| 185 |   supset  ("(_/ \<supset> _)" [50, 51] 50) and
 | |
| 186 |   supset_eq  ("op \<supseteq>") and
 | |
| 187 |   supset_eq  ("(_/ \<supseteq> _)" [50, 51] 50)
 | |
| 188 | ||
| 37387 
3581483cca6c
qualified types "+" and nat; qualified constants Ball, Bex, Suc, curry; modernized some specifications
 haftmann parents: 
36009diff
changeset | 189 | definition Ball :: "'a set \<Rightarrow> ('a \<Rightarrow> bool) \<Rightarrow> bool" where
 | 
| 
3581483cca6c
qualified types "+" and nat; qualified constants Ball, Bex, Suc, curry; modernized some specifications
 haftmann parents: 
36009diff
changeset | 190 | "Ball A P \<longleftrightarrow> (\<forall>x. x \<in> A \<longrightarrow> P x)" -- "bounded universal quantifiers" | 
| 32077 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 191 | |
| 37387 
3581483cca6c
qualified types "+" and nat; qualified constants Ball, Bex, Suc, curry; modernized some specifications
 haftmann parents: 
36009diff
changeset | 192 | definition Bex :: "'a set \<Rightarrow> ('a \<Rightarrow> bool) \<Rightarrow> bool" where
 | 
| 
3581483cca6c
qualified types "+" and nat; qualified constants Ball, Bex, Suc, curry; modernized some specifications
 haftmann parents: 
36009diff
changeset | 193 | "Bex A P \<longleftrightarrow> (\<exists>x. x \<in> A \<and> P x)" -- "bounded existential quantifiers" | 
| 32077 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 194 | |
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 195 | syntax | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 196 |   "_Ball"       :: "pttrn => 'a set => bool => bool"      ("(3ALL _:_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 197 |   "_Bex"        :: "pttrn => 'a set => bool => bool"      ("(3EX _:_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 198 |   "_Bex1"       :: "pttrn => 'a set => bool => bool"      ("(3EX! _:_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 199 |   "_Bleast"     :: "id => 'a set => bool => 'a"           ("(3LEAST _:_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 200 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 201 | syntax (HOL) | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 202 |   "_Ball"       :: "pttrn => 'a set => bool => bool"      ("(3! _:_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 203 |   "_Bex"        :: "pttrn => 'a set => bool => bool"      ("(3? _:_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 204 |   "_Bex1"       :: "pttrn => 'a set => bool => bool"      ("(3?! _:_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 205 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 206 | syntax (xsymbols) | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 207 |   "_Ball"       :: "pttrn => 'a set => bool => bool"      ("(3\<forall>_\<in>_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 208 |   "_Bex"        :: "pttrn => 'a set => bool => bool"      ("(3\<exists>_\<in>_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 209 |   "_Bex1"       :: "pttrn => 'a set => bool => bool"      ("(3\<exists>!_\<in>_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 210 |   "_Bleast"     :: "id => 'a set => bool => 'a"           ("(3LEAST_\<in>_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 211 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 212 | syntax (HTML output) | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 213 |   "_Ball"       :: "pttrn => 'a set => bool => bool"      ("(3\<forall>_\<in>_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 214 |   "_Bex"        :: "pttrn => 'a set => bool => bool"      ("(3\<exists>_\<in>_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 215 |   "_Bex1"       :: "pttrn => 'a set => bool => bool"      ("(3\<exists>!_\<in>_./ _)" [0, 0, 10] 10)
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 216 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 217 | translations | 
| 35115 | 218 | "ALL x:A. P" == "CONST Ball A (%x. P)" | 
| 219 | "EX x:A. P" == "CONST Bex A (%x. P)" | |
| 220 | "EX! x:A. P" => "EX! x. x:A & P" | |
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 221 | "LEAST x:A. P" => "LEAST x. x:A & P" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 222 | |
| 19656 
09be06943252
tuned concrete syntax -- abbreviation/const_syntax;
 wenzelm parents: 
19637diff
changeset | 223 | syntax (output) | 
| 14804 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 224 |   "_setlessAll" :: "[idt, 'a, bool] => bool"  ("(3ALL _<_./ _)"  [0, 0, 10] 10)
 | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 225 |   "_setlessEx"  :: "[idt, 'a, bool] => bool"  ("(3EX _<_./ _)"  [0, 0, 10] 10)
 | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 226 |   "_setleAll"   :: "[idt, 'a, bool] => bool"  ("(3ALL _<=_./ _)" [0, 0, 10] 10)
 | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 227 |   "_setleEx"    :: "[idt, 'a, bool] => bool"  ("(3EX _<=_./ _)" [0, 0, 10] 10)
 | 
| 20217 
25b068a99d2b
linear arithmetic splits certain operators (e.g. min, max, abs)
 webertj parents: 
19870diff
changeset | 228 |   "_setleEx1"   :: "[idt, 'a, bool] => bool"  ("(3EX! _<=_./ _)" [0, 0, 10] 10)
 | 
| 14804 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 229 | |
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 230 | syntax (xsymbols) | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 231 |   "_setlessAll" :: "[idt, 'a, bool] => bool"   ("(3\<forall>_\<subset>_./ _)"  [0, 0, 10] 10)
 | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 232 |   "_setlessEx"  :: "[idt, 'a, bool] => bool"   ("(3\<exists>_\<subset>_./ _)"  [0, 0, 10] 10)
 | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 233 |   "_setleAll"   :: "[idt, 'a, bool] => bool"   ("(3\<forall>_\<subseteq>_./ _)" [0, 0, 10] 10)
 | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 234 |   "_setleEx"    :: "[idt, 'a, bool] => bool"   ("(3\<exists>_\<subseteq>_./ _)" [0, 0, 10] 10)
 | 
| 20217 
25b068a99d2b
linear arithmetic splits certain operators (e.g. min, max, abs)
 webertj parents: 
19870diff
changeset | 235 |   "_setleEx1"   :: "[idt, 'a, bool] => bool"   ("(3\<exists>!_\<subseteq>_./ _)" [0, 0, 10] 10)
 | 
| 14804 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 236 | |
| 19656 
09be06943252
tuned concrete syntax -- abbreviation/const_syntax;
 wenzelm parents: 
19637diff
changeset | 237 | syntax (HOL output) | 
| 14804 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 238 |   "_setlessAll" :: "[idt, 'a, bool] => bool"   ("(3! _<_./ _)"  [0, 0, 10] 10)
 | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 239 |   "_setlessEx"  :: "[idt, 'a, bool] => bool"   ("(3? _<_./ _)"  [0, 0, 10] 10)
 | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 240 |   "_setleAll"   :: "[idt, 'a, bool] => bool"   ("(3! _<=_./ _)" [0, 0, 10] 10)
 | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 241 |   "_setleEx"    :: "[idt, 'a, bool] => bool"   ("(3? _<=_./ _)" [0, 0, 10] 10)
 | 
| 20217 
25b068a99d2b
linear arithmetic splits certain operators (e.g. min, max, abs)
 webertj parents: 
19870diff
changeset | 242 |   "_setleEx1"   :: "[idt, 'a, bool] => bool"   ("(3?! _<=_./ _)" [0, 0, 10] 10)
 | 
| 14804 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 243 | |
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 244 | syntax (HTML output) | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 245 |   "_setlessAll" :: "[idt, 'a, bool] => bool"   ("(3\<forall>_\<subset>_./ _)"  [0, 0, 10] 10)
 | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 246 |   "_setlessEx"  :: "[idt, 'a, bool] => bool"   ("(3\<exists>_\<subset>_./ _)"  [0, 0, 10] 10)
 | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 247 |   "_setleAll"   :: "[idt, 'a, bool] => bool"   ("(3\<forall>_\<subseteq>_./ _)" [0, 0, 10] 10)
 | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 248 |   "_setleEx"    :: "[idt, 'a, bool] => bool"   ("(3\<exists>_\<subseteq>_./ _)" [0, 0, 10] 10)
 | 
| 20217 
25b068a99d2b
linear arithmetic splits certain operators (e.g. min, max, abs)
 webertj parents: 
19870diff
changeset | 249 |   "_setleEx1"   :: "[idt, 'a, bool] => bool"   ("(3\<exists>!_\<subseteq>_./ _)" [0, 0, 10] 10)
 | 
| 14804 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 250 | |
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 251 | translations | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 252 | "\<forall>A\<subset>B. P" => "ALL A. A \<subset> B --> P" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 253 | "\<exists>A\<subset>B. P" => "EX A. A \<subset> B & P" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 254 | "\<forall>A\<subseteq>B. P" => "ALL A. A \<subseteq> B --> P" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 255 | "\<exists>A\<subseteq>B. P" => "EX A. A \<subseteq> B & P" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 256 | "\<exists>!A\<subseteq>B. P" => "EX! A. A \<subseteq> B & P" | 
| 14804 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 257 | |
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 258 | print_translation {*
 | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 259 | let | 
| 42287 
d98eb048a2e4
discontinued special treatment of structure Mixfix;
 wenzelm parents: 
42284diff
changeset | 260 |   val All_binder = Mixfix.binder_name @{const_syntax All};
 | 
| 
d98eb048a2e4
discontinued special treatment of structure Mixfix;
 wenzelm parents: 
42284diff
changeset | 261 |   val Ex_binder = Mixfix.binder_name @{const_syntax Ex};
 | 
| 38786 
e46e7a9cb622
formerly unnamed infix impliciation now named HOL.implies
 haftmann parents: 
38715diff
changeset | 262 |   val impl = @{const_syntax HOL.implies};
 | 
| 38795 
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
 haftmann parents: 
38786diff
changeset | 263 |   val conj = @{const_syntax HOL.conj};
 | 
| 35115 | 264 |   val sbset = @{const_syntax subset};
 | 
| 265 |   val sbset_eq = @{const_syntax subset_eq};
 | |
| 21819 | 266 | |
| 267 | val trans = | |
| 35115 | 268 |    [((All_binder, impl, sbset), @{syntax_const "_setlessAll"}),
 | 
| 269 |     ((All_binder, impl, sbset_eq), @{syntax_const "_setleAll"}),
 | |
| 270 |     ((Ex_binder, conj, sbset), @{syntax_const "_setlessEx"}),
 | |
| 271 |     ((Ex_binder, conj, sbset_eq), @{syntax_const "_setleEx"})];
 | |
| 21819 | 272 | |
| 273 | fun mk v v' c n P = | |
| 274 | if v = v' andalso not (Term.exists_subterm (fn Free (x, _) => x = v | _ => false) n) | |
| 42284 | 275 | then Syntax.const c $ Syntax_Trans.mark_bound v' $ n $ P else raise Match; | 
| 21819 | 276 | |
| 277 | fun tr' q = (q, | |
| 46137 
0477785525be
tuned -- more direct @{type_name set} (NB: binder_tr' retains the original non-syntax type for the bound/free variable);
 wenzelm parents: 
46128diff
changeset | 278 |         fn [Const (@{syntax_const "_bound"}, _) $ Free (v, Type (@{type_name set}, _)),
 | 
| 35115 | 279 | Const (c, _) $ | 
| 280 |               (Const (d, _) $ (Const (@{syntax_const "_bound"}, _) $ Free (v', _)) $ n) $ P] =>
 | |
| 46137 
0477785525be
tuned -- more direct @{type_name set} (NB: binder_tr' retains the original non-syntax type for the bound/free variable);
 wenzelm parents: 
46128diff
changeset | 281 | (case AList.lookup (op =) trans (q, c, d) of | 
| 
0477785525be
tuned -- more direct @{type_name set} (NB: binder_tr' retains the original non-syntax type for the bound/free variable);
 wenzelm parents: 
46128diff
changeset | 282 | NONE => raise Match | 
| 
0477785525be
tuned -- more direct @{type_name set} (NB: binder_tr' retains the original non-syntax type for the bound/free variable);
 wenzelm parents: 
46128diff
changeset | 283 | | SOME l => mk v v' l n P) | 
| 35115 | 284 | | _ => raise Match); | 
| 14804 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 285 | in | 
| 21819 | 286 | [tr' All_binder, tr' Ex_binder] | 
| 14804 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 287 | end | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 288 | *} | 
| 
8de39d3e8eb6
Corrected printer bug for bounded quantifiers Q x<=y. P
 nipkow parents: 
14752diff
changeset | 289 | |
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 290 | |
| 11979 | 291 | text {*
 | 
| 292 |   \medskip Translate between @{text "{e | x1...xn. P}"} and @{text
 | |
| 293 |   "{u. EX x1..xn. u = e & P}"}; @{text "{y. EX x1..xn. y = e & P}"} is
 | |
| 294 |   only translated if @{text "[0..n] subset bvs(e)"}.
 | |
| 295 | *} | |
| 296 | ||
| 35115 | 297 | syntax | 
| 298 |   "_Setcompr" :: "'a => idts => bool => 'a set"    ("(1{_ |/_./ _})")
 | |
| 299 | ||
| 11979 | 300 | parse_translation {*
 | 
| 301 | let | |
| 42284 | 302 |     val ex_tr = snd (Syntax_Trans.mk_binder_tr ("EX ", @{const_syntax Ex}));
 | 
| 3947 | 303 | |
| 35115 | 304 |     fun nvars (Const (@{syntax_const "_idts"}, _) $ _ $ idts) = nvars idts + 1
 | 
| 11979 | 305 | | nvars _ = 1; | 
| 306 | ||
| 307 | fun setcompr_tr [e, idts, b] = | |
| 308 | let | |
| 38864 
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
 haftmann parents: 
38795diff
changeset | 309 |         val eq = Syntax.const @{const_syntax HOL.eq} $ Bound (nvars idts) $ e;
 | 
| 38795 
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
 haftmann parents: 
38786diff
changeset | 310 |         val P = Syntax.const @{const_syntax HOL.conj} $ eq $ b;
 | 
| 11979 | 311 | val exP = ex_tr [idts, P]; | 
| 44241 | 312 |       in Syntax.const @{const_syntax Collect} $ absdummy dummyT exP end;
 | 
| 11979 | 313 | |
| 35115 | 314 |   in [(@{syntax_const "_Setcompr"}, setcompr_tr)] end;
 | 
| 11979 | 315 | *} | 
| 923 | 316 | |
| 35115 | 317 | print_translation {*
 | 
| 42284 | 318 |  [Syntax_Trans.preserve_binder_abs2_tr' @{const_syntax Ball} @{syntax_const "_Ball"},
 | 
| 319 |   Syntax_Trans.preserve_binder_abs2_tr' @{const_syntax Bex} @{syntax_const "_Bex"}]
 | |
| 35115 | 320 | *} -- {* to avoid eta-contraction of body *}
 | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 321 | |
| 13763 
f94b569cd610
added print translations tha avoid eta contraction for important binders.
 nipkow parents: 
13653diff
changeset | 322 | print_translation {*
 | 
| 
f94b569cd610
added print translations tha avoid eta contraction for important binders.
 nipkow parents: 
13653diff
changeset | 323 | let | 
| 42284 | 324 |   val ex_tr' = snd (Syntax_Trans.mk_binder_tr' (@{const_syntax Ex}, "DUMMY"));
 | 
| 13763 
f94b569cd610
added print translations tha avoid eta contraction for important binders.
 nipkow parents: 
13653diff
changeset | 325 | |
| 
f94b569cd610
added print translations tha avoid eta contraction for important binders.
 nipkow parents: 
13653diff
changeset | 326 | fun setcompr_tr' [Abs (abs as (_, _, P))] = | 
| 
f94b569cd610
added print translations tha avoid eta contraction for important binders.
 nipkow parents: 
13653diff
changeset | 327 | let | 
| 35115 | 328 |       fun check (Const (@{const_syntax Ex}, _) $ Abs (_, _, P), n) = check (P, n + 1)
 | 
| 38795 
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
 haftmann parents: 
38786diff
changeset | 329 |         | check (Const (@{const_syntax HOL.conj}, _) $
 | 
| 38864 
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
 haftmann parents: 
38795diff
changeset | 330 |               (Const (@{const_syntax HOL.eq}, _) $ Bound m $ e) $ P, n) =
 | 
| 13763 
f94b569cd610
added print translations tha avoid eta contraction for important binders.
 nipkow parents: 
13653diff
changeset | 331 | n > 0 andalso m = n andalso not (loose_bvar1 (P, n)) andalso | 
| 33038 | 332 | subset (op =) (0 upto (n - 1), add_loose_bnos (e, 0, [])) | 
| 35115 | 333 | | check _ = false; | 
| 923 | 334 | |
| 11979 | 335 | fun tr' (_ $ abs) = | 
| 336 | let val _ $ idts $ (_ $ (_ $ _ $ e) $ Q) = ex_tr' [abs] | |
| 35115 | 337 |           in Syntax.const @{syntax_const "_Setcompr"} $ e $ idts $ Q end;
 | 
| 338 | in | |
| 339 | if check (P, 0) then tr' P | |
| 340 | else | |
| 341 | let | |
| 42284 | 342 | val (x as _ $ Free(xN, _), t) = Syntax_Trans.atomic_abs_tr' abs; | 
| 35115 | 343 |           val M = Syntax.const @{syntax_const "_Coll"} $ x $ t;
 | 
| 344 | in | |
| 345 | case t of | |
| 38795 
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
 haftmann parents: 
38786diff
changeset | 346 |             Const (@{const_syntax HOL.conj}, _) $
 | 
| 37677 | 347 |               (Const (@{const_syntax Set.member}, _) $
 | 
| 35115 | 348 |                 (Const (@{syntax_const "_bound"}, _) $ Free (yN, _)) $ A) $ P =>
 | 
| 349 |             if xN = yN then Syntax.const @{syntax_const "_Collect"} $ x $ A $ P else M
 | |
| 350 | | _ => M | |
| 351 | end | |
| 13763 
f94b569cd610
added print translations tha avoid eta contraction for important binders.
 nipkow parents: 
13653diff
changeset | 352 | end; | 
| 35115 | 353 |   in [(@{const_syntax Collect}, setcompr_tr')] end;
 | 
| 11979 | 354 | *} | 
| 355 | ||
| 42455 | 356 | simproc_setup defined_Bex ("EX x:A. P x & Q x") = {*
 | 
| 357 | let | |
| 358 |     val unfold_bex_tac = unfold_tac @{thms Bex_def};
 | |
| 359 | fun prove_bex_tac ss = unfold_bex_tac ss THEN Quantifier1.prove_one_point_ex_tac; | |
| 42459 | 360 | in fn _ => fn ss => Quantifier1.rearrange_bex (prove_bex_tac ss) ss end | 
| 42455 | 361 | *} | 
| 362 | ||
| 363 | simproc_setup defined_All ("ALL x:A. P x --> Q x") = {*
 | |
| 364 | let | |
| 365 |     val unfold_ball_tac = unfold_tac @{thms Ball_def};
 | |
| 366 | fun prove_ball_tac ss = unfold_ball_tac ss THEN Quantifier1.prove_one_point_all_tac; | |
| 42459 | 367 | in fn _ => fn ss => Quantifier1.rearrange_ball (prove_ball_tac ss) ss end | 
| 32117 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 368 | *} | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 369 | |
| 11979 | 370 | lemma ballI [intro!]: "(!!x. x:A ==> P x) ==> ALL x:A. P x" | 
| 371 | by (simp add: Ball_def) | |
| 372 | ||
| 373 | lemmas strip = impI allI ballI | |
| 374 | ||
| 375 | lemma bspec [dest?]: "ALL x:A. P x ==> x:A ==> P x" | |
| 376 | by (simp add: Ball_def) | |
| 377 | ||
| 378 | text {*
 | |
| 379 | Gives better instantiation for bound: | |
| 380 | *} | |
| 381 | ||
| 26339 | 382 | declaration {* fn _ =>
 | 
| 46459 | 383 |   Classical.map_cs (fn cs => cs addbefore ("bspec", dtac @{thm bspec} THEN' assume_tac))
 | 
| 11979 | 384 | *} | 
| 385 | ||
| 32117 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 386 | ML {*
 | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 387 | structure Simpdata = | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 388 | struct | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 389 | |
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 390 | open Simpdata; | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 391 | |
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 392 | val mksimps_pairs = [(@{const_name Ball}, @{thms bspec})] @ mksimps_pairs;
 | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 393 | |
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 394 | end; | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 395 | |
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 396 | open Simpdata; | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 397 | *} | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 398 | |
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 399 | declaration {* fn _ =>
 | 
| 45625 
750c5a47400b
modernized some old-style infix operations, which were left over from the time of ML proof scripts;
 wenzelm parents: 
45607diff
changeset | 400 | Simplifier.map_ss (Simplifier.set_mksimps (mksimps mksimps_pairs)) | 
| 32117 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 401 | *} | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 402 | |
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 403 | lemma ballE [elim]: "ALL x:A. P x ==> (P x ==> Q) ==> (x ~: A ==> Q) ==> Q" | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 404 | by (unfold Ball_def) blast | 
| 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 405 | |
| 11979 | 406 | lemma bexI [intro]: "P x ==> x:A ==> EX x:A. P x" | 
| 407 |   -- {* Normally the best argument order: @{prop "P x"} constrains the
 | |
| 408 |     choice of @{prop "x:A"}. *}
 | |
| 409 | by (unfold Bex_def) blast | |
| 410 | ||
| 13113 | 411 | lemma rev_bexI [intro?]: "x:A ==> P x ==> EX x:A. P x" | 
| 11979 | 412 |   -- {* The best argument order when there is only one @{prop "x:A"}. *}
 | 
| 413 | by (unfold Bex_def) blast | |
| 414 | ||
| 415 | lemma bexCI: "(ALL x:A. ~P x ==> P a) ==> a:A ==> EX x:A. P x" | |
| 416 | by (unfold Bex_def) blast | |
| 417 | ||
| 418 | lemma bexE [elim!]: "EX x:A. P x ==> (!!x. x:A ==> P x ==> Q) ==> Q" | |
| 419 | by (unfold Bex_def) blast | |
| 420 | ||
| 421 | lemma ball_triv [simp]: "(ALL x:A. P) = ((EX x. x:A) --> P)" | |
| 422 |   -- {* Trival rewrite rule. *}
 | |
| 423 | by (simp add: Ball_def) | |
| 424 | ||
| 425 | lemma bex_triv [simp]: "(EX x:A. P) = ((EX x. x:A) & P)" | |
| 426 |   -- {* Dual form for existentials. *}
 | |
| 427 | by (simp add: Bex_def) | |
| 428 | ||
| 429 | lemma bex_triv_one_point1 [simp]: "(EX x:A. x = a) = (a:A)" | |
| 430 | by blast | |
| 431 | ||
| 432 | lemma bex_triv_one_point2 [simp]: "(EX x:A. a = x) = (a:A)" | |
| 433 | by blast | |
| 434 | ||
| 435 | lemma bex_one_point1 [simp]: "(EX x:A. x = a & P x) = (a:A & P a)" | |
| 436 | by blast | |
| 437 | ||
| 438 | lemma bex_one_point2 [simp]: "(EX x:A. a = x & P x) = (a:A & P a)" | |
| 439 | by blast | |
| 440 | ||
| 441 | lemma ball_one_point1 [simp]: "(ALL x:A. x = a --> P x) = (a:A --> P a)" | |
| 442 | by blast | |
| 443 | ||
| 444 | lemma ball_one_point2 [simp]: "(ALL x:A. a = x --> P x) = (a:A --> P a)" | |
| 445 | by blast | |
| 446 | ||
| 43818 | 447 | lemma ball_conj_distrib: | 
| 448 | "(\<forall>x\<in>A. P x \<and> Q x) \<longleftrightarrow> ((\<forall>x\<in>A. P x) \<and> (\<forall>x\<in>A. Q x))" | |
| 449 | by blast | |
| 450 | ||
| 451 | lemma bex_disj_distrib: | |
| 452 | "(\<exists>x\<in>A. P x \<or> Q x) \<longleftrightarrow> ((\<exists>x\<in>A. P x) \<or> (\<exists>x\<in>A. Q x))" | |
| 453 | by blast | |
| 454 | ||
| 11979 | 455 | |
| 32081 | 456 | text {* Congruence rules *}
 | 
| 11979 | 457 | |
| 16636 
1ed737a98198
Added strong_ball_cong and strong_bex_cong (these are now the standard
 berghofe parents: 
15950diff
changeset | 458 | lemma ball_cong: | 
| 11979 | 459 | "A = B ==> (!!x. x:B ==> P x = Q x) ==> | 
| 460 | (ALL x:A. P x) = (ALL x:B. Q x)" | |
| 461 | by (simp add: Ball_def) | |
| 462 | ||
| 16636 
1ed737a98198
Added strong_ball_cong and strong_bex_cong (these are now the standard
 berghofe parents: 
15950diff
changeset | 463 | lemma strong_ball_cong [cong]: | 
| 
1ed737a98198
Added strong_ball_cong and strong_bex_cong (these are now the standard
 berghofe parents: 
15950diff
changeset | 464 | "A = B ==> (!!x. x:B =simp=> P x = Q x) ==> | 
| 
1ed737a98198
Added strong_ball_cong and strong_bex_cong (these are now the standard
 berghofe parents: 
15950diff
changeset | 465 | (ALL x:A. P x) = (ALL x:B. Q x)" | 
| 
1ed737a98198
Added strong_ball_cong and strong_bex_cong (these are now the standard
 berghofe parents: 
15950diff
changeset | 466 | by (simp add: simp_implies_def Ball_def) | 
| 
1ed737a98198
Added strong_ball_cong and strong_bex_cong (these are now the standard
 berghofe parents: 
15950diff
changeset | 467 | |
| 
1ed737a98198
Added strong_ball_cong and strong_bex_cong (these are now the standard
 berghofe parents: 
15950diff
changeset | 468 | lemma bex_cong: | 
| 11979 | 469 | "A = B ==> (!!x. x:B ==> P x = Q x) ==> | 
| 470 | (EX x:A. P x) = (EX x:B. Q x)" | |
| 471 | by (simp add: Bex_def cong: conj_cong) | |
| 1273 | 472 | |
| 16636 
1ed737a98198
Added strong_ball_cong and strong_bex_cong (these are now the standard
 berghofe parents: 
15950diff
changeset | 473 | lemma strong_bex_cong [cong]: | 
| 
1ed737a98198
Added strong_ball_cong and strong_bex_cong (these are now the standard
 berghofe parents: 
15950diff
changeset | 474 | "A = B ==> (!!x. x:B =simp=> P x = Q x) ==> | 
| 
1ed737a98198
Added strong_ball_cong and strong_bex_cong (these are now the standard
 berghofe parents: 
15950diff
changeset | 475 | (EX x:A. P x) = (EX x:B. Q x)" | 
| 
1ed737a98198
Added strong_ball_cong and strong_bex_cong (these are now the standard
 berghofe parents: 
15950diff
changeset | 476 | by (simp add: simp_implies_def Bex_def cong: conj_cong) | 
| 
1ed737a98198
Added strong_ball_cong and strong_bex_cong (these are now the standard
 berghofe parents: 
15950diff
changeset | 477 | |
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 478 | |
| 32081 | 479 | subsection {* Basic operations *}
 | 
| 480 | ||
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 481 | subsubsection {* Subsets *}
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 482 | |
| 33022 
c95102496490
 Removal of the unused atpset concept, the atp attribute and some related code.
 paulson parents: 
32888diff
changeset | 483 | lemma subsetI [intro!]: "(\<And>x. x \<in> A \<Longrightarrow> x \<in> B) \<Longrightarrow> A \<subseteq> B" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 484 | by (simp add: less_eq_set_def le_fun_def) | 
| 30352 | 485 | |
| 11979 | 486 | text {*
 | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 487 |   \medskip Map the type @{text "'a set => anything"} to just @{typ
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 488 |   'a}; for overloading constants whose first argument has type @{typ
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 489 | "'a set"}. | 
| 11979 | 490 | *} | 
| 491 | ||
| 30596 | 492 | lemma subsetD [elim, intro?]: "A \<subseteq> B ==> c \<in> A ==> c \<in> B" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 493 | by (simp add: less_eq_set_def le_fun_def) | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 494 |   -- {* Rule in Modus Ponens style. *}
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 495 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 496 | lemma rev_subsetD [no_atp,intro?]: "c \<in> A ==> A \<subseteq> B ==> c \<in> B" | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 497 |   -- {* The same, with reversed premises for use with @{text erule} --
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 498 |       cf @{text rev_mp}. *}
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 499 | by (rule subsetD) | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 500 | |
| 11979 | 501 | text {*
 | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 502 |   \medskip Converts @{prop "A \<subseteq> B"} to @{prop "x \<in> A ==> x \<in> B"}.
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 503 | *} | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 504 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 505 | lemma subsetCE [no_atp,elim]: "A \<subseteq> B ==> (c \<notin> A ==> P) ==> (c \<in> B ==> P) ==> P" | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 506 |   -- {* Classical elimination rule. *}
 | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 507 | by (auto simp add: less_eq_set_def le_fun_def) | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 508 | |
| 47398 | 509 | lemma subset_eq [no_atp]: "A \<le> B = (\<forall>x\<in>A. x \<in> B)" by blast | 
| 2388 | 510 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 511 | lemma contra_subsetD [no_atp]: "A \<subseteq> B ==> c \<notin> B ==> c \<notin> A" | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 512 | by blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 513 | |
| 45121 | 514 | lemma subset_refl: "A \<subseteq> A" | 
| 515 | by (fact order_refl) (* already [iff] *) | |
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 516 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 517 | lemma subset_trans: "A \<subseteq> B ==> B \<subseteq> C ==> A \<subseteq> C" | 
| 32081 | 518 | by (fact order_trans) | 
| 519 | ||
| 520 | lemma set_rev_mp: "x:A ==> A \<subseteq> B ==> x:B" | |
| 521 | by (rule subsetD) | |
| 522 | ||
| 523 | lemma set_mp: "A \<subseteq> B ==> x:A ==> x:B" | |
| 524 | by (rule subsetD) | |
| 525 | ||
| 46146 
6baea4fca6bd
incorporated various theorems from theory More_Set into corpus
 haftmann parents: 
46137diff
changeset | 526 | lemma subset_not_subset_eq [code]: | 
| 
6baea4fca6bd
incorporated various theorems from theory More_Set into corpus
 haftmann parents: 
46137diff
changeset | 527 | "A \<subset> B \<longleftrightarrow> A \<subseteq> B \<and> \<not> B \<subseteq> A" | 
| 
6baea4fca6bd
incorporated various theorems from theory More_Set into corpus
 haftmann parents: 
46137diff
changeset | 528 | by (fact less_le_not_le) | 
| 
6baea4fca6bd
incorporated various theorems from theory More_Set into corpus
 haftmann parents: 
46137diff
changeset | 529 | |
| 33044 | 530 | lemma eq_mem_trans: "a=b ==> b \<in> A ==> a \<in> A" | 
| 531 | by simp | |
| 532 | ||
| 32081 | 533 | lemmas basic_trans_rules [trans] = | 
| 33044 | 534 | order_trans_rules set_rev_mp set_mp eq_mem_trans | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 535 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 536 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 537 | subsubsection {* Equality *}
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 538 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 539 | lemma subset_antisym [intro!]: "A \<subseteq> B ==> B \<subseteq> A ==> A = B" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 540 |   -- {* Anti-symmetry of the subset relation. *}
 | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39213diff
changeset | 541 | by (iprover intro: set_eqI subsetD) | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 542 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 543 | text {*
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 544 | \medskip Equality rules from ZF set theory -- are they appropriate | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 545 | here? | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 546 | *} | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 547 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 548 | lemma equalityD1: "A = B ==> A \<subseteq> B" | 
| 34209 | 549 | by simp | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 550 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 551 | lemma equalityD2: "A = B ==> B \<subseteq> A" | 
| 34209 | 552 | by simp | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 553 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 554 | text {*
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 555 |   \medskip Be careful when adding this to the claset as @{text
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 556 |   subset_empty} is in the simpset: @{prop "A = {}"} goes to @{prop "{}
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 557 |   \<subseteq> A"} and @{prop "A \<subseteq> {}"} and then back to @{prop "A = {}"}!
 | 
| 30352 | 558 | *} | 
| 559 | ||
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 560 | lemma equalityE: "A = B ==> (A \<subseteq> B ==> B \<subseteq> A ==> P) ==> P" | 
| 34209 | 561 | by simp | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 562 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 563 | lemma equalityCE [elim]: | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 564 | "A = B ==> (c \<in> A ==> c \<in> B ==> P) ==> (c \<notin> A ==> c \<notin> B ==> P) ==> P" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 565 | by blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 566 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 567 | lemma eqset_imp_iff: "A = B ==> (x : A) = (x : B)" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 568 | by simp | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 569 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 570 | lemma eqelem_imp_iff: "x = y ==> (x : A) = (y : A)" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 571 | by simp | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 572 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 573 | |
| 41082 | 574 | subsubsection {* The empty set *}
 | 
| 575 | ||
| 576 | lemma empty_def: | |
| 577 |   "{} = {x. False}"
 | |
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 578 | by (simp add: bot_set_def bot_fun_def) | 
| 41082 | 579 | |
| 580 | lemma empty_iff [simp]: "(c : {}) = False"
 | |
| 581 | by (simp add: empty_def) | |
| 582 | ||
| 583 | lemma emptyE [elim!]: "a : {} ==> P"
 | |
| 584 | by simp | |
| 585 | ||
| 586 | lemma empty_subsetI [iff]: "{} \<subseteq> A"
 | |
| 587 |     -- {* One effect is to delete the ASSUMPTION @{prop "{} <= A"} *}
 | |
| 588 | by blast | |
| 589 | ||
| 590 | lemma equals0I: "(!!y. y \<in> A ==> False) ==> A = {}"
 | |
| 591 | by blast | |
| 592 | ||
| 593 | lemma equals0D: "A = {} ==> a \<notin> A"
 | |
| 594 |     -- {* Use for reasoning about disjointness: @{text "A Int B = {}"} *}
 | |
| 595 | by blast | |
| 596 | ||
| 597 | lemma ball_empty [simp]: "Ball {} P = True"
 | |
| 598 | by (simp add: Ball_def) | |
| 599 | ||
| 600 | lemma bex_empty [simp]: "Bex {} P = False"
 | |
| 601 | by (simp add: Bex_def) | |
| 602 | ||
| 603 | ||
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 604 | subsubsection {* The universal set -- UNIV *}
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 605 | |
| 32264 
0be31453f698
Set.UNIV and Set.empty are mere abbreviations for top and bot
 haftmann parents: 
32139diff
changeset | 606 | abbreviation UNIV :: "'a set" where | 
| 
0be31453f698
Set.UNIV and Set.empty are mere abbreviations for top and bot
 haftmann parents: 
32139diff
changeset | 607 | "UNIV \<equiv> top" | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 608 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 609 | lemma UNIV_def: | 
| 32117 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 610 |   "UNIV = {x. True}"
 | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 611 | by (simp add: top_set_def top_fun_def) | 
| 32081 | 612 | |
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 613 | lemma UNIV_I [simp]: "x : UNIV" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 614 | by (simp add: UNIV_def) | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 615 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 616 | declare UNIV_I [intro]  -- {* unsafe makes it less likely to cause problems *}
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 617 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 618 | lemma UNIV_witness [intro?]: "EX x. x : UNIV" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 619 | by simp | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 620 | |
| 45121 | 621 | lemma subset_UNIV: "A \<subseteq> UNIV" | 
| 622 | by (fact top_greatest) (* already simp *) | |
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 623 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 624 | text {*
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 625 |   \medskip Eta-contracting these two rules (to remove @{text P})
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 626 | causes them to be ignored because of their interaction with | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 627 | congruence rules. | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 628 | *} | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 629 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 630 | lemma ball_UNIV [simp]: "Ball UNIV P = All P" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 631 | by (simp add: Ball_def) | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 632 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 633 | lemma bex_UNIV [simp]: "Bex UNIV P = Ex P" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 634 | by (simp add: Bex_def) | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 635 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 636 | lemma UNIV_eq_I: "(\<And>x. x \<in> A) \<Longrightarrow> UNIV = A" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 637 | by auto | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 638 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 639 | lemma UNIV_not_empty [iff]: "UNIV ~= {}"
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 640 | by (blast elim: equalityE) | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 641 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 642 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 643 | subsubsection {* The Powerset operator -- Pow *}
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 644 | |
| 32077 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 645 | definition Pow :: "'a set => 'a set set" where | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 646 |   Pow_def: "Pow A = {B. B \<le> A}"
 | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 647 | |
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 648 | lemma Pow_iff [iff]: "(A \<in> Pow B) = (A \<subseteq> B)" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 649 | by (simp add: Pow_def) | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 650 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 651 | lemma PowI: "A \<subseteq> B ==> A \<in> Pow B" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 652 | by (simp add: Pow_def) | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 653 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 654 | lemma PowD: "A \<in> Pow B ==> A \<subseteq> B" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 655 | by (simp add: Pow_def) | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 656 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 657 | lemma Pow_bottom: "{} \<in> Pow B"
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 658 | by simp | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 659 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 660 | lemma Pow_top: "A \<in> Pow A" | 
| 34209 | 661 | by simp | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 662 | |
| 40703 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 663 | lemma Pow_not_empty: "Pow A \<noteq> {}"
 | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 664 | using Pow_top by blast | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 665 | |
| 41076 
a7fba340058c
primitive definitions of bot/top/inf/sup for bool and fun are named with canonical suffix `_def` rather than `_eq`;
 haftmann parents: 
40872diff
changeset | 666 | |
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 667 | subsubsection {* Set complement *}
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 668 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 669 | lemma Compl_iff [simp]: "(c \<in> -A) = (c \<notin> A)" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 670 | by (simp add: fun_Compl_def uminus_set_def) | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 671 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 672 | lemma ComplI [intro!]: "(c \<in> A ==> False) ==> c \<in> -A" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 673 | by (simp add: fun_Compl_def uminus_set_def) blast | 
| 923 | 674 | |
| 11979 | 675 | text {*
 | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 676 | \medskip This form, with negated conclusion, works well with the | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 677 | Classical prover. Negated assumptions behave like formulae on the | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 678 | right side of the notional turnstile ... *} | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 679 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 680 | lemma ComplD [dest!]: "c : -A ==> c~:A" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 681 | by simp | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 682 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 683 | lemmas ComplE = ComplD [elim_format] | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 684 | |
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 685 | lemma Compl_eq: "- A = {x. ~ x : A}"
 | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 686 | by blast | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 687 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 688 | |
| 41082 | 689 | subsubsection {* Binary intersection *}
 | 
| 690 | ||
| 691 | abbreviation inter :: "'a set \<Rightarrow> 'a set \<Rightarrow> 'a set" (infixl "Int" 70) where | |
| 692 | "op Int \<equiv> inf" | |
| 693 | ||
| 694 | notation (xsymbols) | |
| 695 | inter (infixl "\<inter>" 70) | |
| 696 | ||
| 697 | notation (HTML output) | |
| 698 | inter (infixl "\<inter>" 70) | |
| 699 | ||
| 700 | lemma Int_def: | |
| 701 |   "A \<inter> B = {x. x \<in> A \<and> x \<in> B}"
 | |
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 702 | by (simp add: inf_set_def inf_fun_def) | 
| 41082 | 703 | |
| 704 | lemma Int_iff [simp]: "(c : A Int B) = (c:A & c:B)" | |
| 705 | by (unfold Int_def) blast | |
| 706 | ||
| 707 | lemma IntI [intro!]: "c:A ==> c:B ==> c : A Int B" | |
| 708 | by simp | |
| 709 | ||
| 710 | lemma IntD1: "c : A Int B ==> c:A" | |
| 711 | by simp | |
| 712 | ||
| 713 | lemma IntD2: "c : A Int B ==> c:B" | |
| 714 | by simp | |
| 715 | ||
| 716 | lemma IntE [elim!]: "c : A Int B ==> (c:A ==> c:B ==> P) ==> P" | |
| 717 | by simp | |
| 718 | ||
| 719 | lemma mono_Int: "mono f \<Longrightarrow> f (A \<inter> B) \<subseteq> f A \<inter> f B" | |
| 720 | by (fact mono_inf) | |
| 721 | ||
| 722 | ||
| 723 | subsubsection {* Binary union *}
 | |
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 724 | |
| 32683 
7c1fe854ca6a
inter and union are mere abbreviations for inf and sup
 haftmann parents: 
32456diff
changeset | 725 | abbreviation union :: "'a set \<Rightarrow> 'a set \<Rightarrow> 'a set" (infixl "Un" 65) where | 
| 41076 
a7fba340058c
primitive definitions of bot/top/inf/sup for bool and fun are named with canonical suffix `_def` rather than `_eq`;
 haftmann parents: 
40872diff
changeset | 726 | "union \<equiv> sup" | 
| 32081 | 727 | |
| 728 | notation (xsymbols) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 729 | union (infixl "\<union>" 65) | 
| 32081 | 730 | |
| 731 | notation (HTML output) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 732 | union (infixl "\<union>" 65) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 733 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 734 | lemma Un_def: | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 735 |   "A \<union> B = {x. x \<in> A \<or> x \<in> B}"
 | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 736 | by (simp add: sup_set_def sup_fun_def) | 
| 32081 | 737 | |
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 738 | lemma Un_iff [simp]: "(c : A Un B) = (c:A | c:B)" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 739 | by (unfold Un_def) blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 740 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 741 | lemma UnI1 [elim?]: "c:A ==> c : A Un B" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 742 | by simp | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 743 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 744 | lemma UnI2 [elim?]: "c:B ==> c : A Un B" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 745 | by simp | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 746 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 747 | text {*
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 748 |   \medskip Classical introduction rule: no commitment to @{prop A} vs
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 749 |   @{prop B}.
 | 
| 11979 | 750 | *} | 
| 751 | ||
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 752 | lemma UnCI [intro!]: "(c~:B ==> c:A) ==> c : A Un B" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 753 | by auto | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 754 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 755 | lemma UnE [elim!]: "c : A Un B ==> (c:A ==> P) ==> (c:B ==> P) ==> P" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 756 | by (unfold Un_def) blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 757 | |
| 32117 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 758 | lemma insert_def: "insert a B = {x. x = a} \<union> B"
 | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 759 | by (simp add: insert_compr Un_def) | 
| 32081 | 760 | |
| 761 | lemma mono_Un: "mono f \<Longrightarrow> f A \<union> f B \<subseteq> f (A \<union> B)" | |
| 32683 
7c1fe854ca6a
inter and union are mere abbreviations for inf and sup
 haftmann parents: 
32456diff
changeset | 762 | by (fact mono_sup) | 
| 32081 | 763 | |
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 764 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 765 | subsubsection {* Set difference *}
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 766 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 767 | lemma Diff_iff [simp]: "(c : A - B) = (c:A & c~:B)" | 
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 768 | by (simp add: minus_set_def fun_diff_def) | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 769 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 770 | lemma DiffI [intro!]: "c : A ==> c ~: B ==> c : A - B" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 771 | by simp | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 772 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 773 | lemma DiffD1: "c : A - B ==> c : A" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 774 | by simp | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 775 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 776 | lemma DiffD2: "c : A - B ==> c : B ==> P" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 777 | by simp | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 778 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 779 | lemma DiffE [elim!]: "c : A - B ==> (c:A ==> c~:B ==> P) ==> P" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 780 | by simp | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 781 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 782 | lemma set_diff_eq: "A - B = {x. x : A & ~ x : B}" by blast
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 783 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 784 | lemma Compl_eq_Diff_UNIV: "-A = (UNIV - A)" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 785 | by blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 786 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 787 | |
| 31456 | 788 | subsubsection {* Augmenting a set -- @{const insert} *}
 | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 789 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 790 | lemma insert_iff [simp]: "(a : insert b A) = (a = b | a:A)" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 791 | by (unfold insert_def) blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 792 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 793 | lemma insertI1: "a : insert a B" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 794 | by simp | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 795 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 796 | lemma insertI2: "a : B ==> a : insert b B" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 797 | by simp | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 798 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 799 | lemma insertE [elim!]: "a : insert b A ==> (a = b ==> P) ==> (a:A ==> P) ==> P" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 800 | by (unfold insert_def) blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 801 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 802 | lemma insertCI [intro!]: "(a~:B ==> a = b) ==> a: insert b B" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 803 |   -- {* Classical introduction rule. *}
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 804 | by auto | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 805 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 806 | lemma subset_insert_iff: "(A \<subseteq> insert x B) = (if x:A then A - {x} \<subseteq> B else A \<subseteq> B)"
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 807 | by auto | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 808 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 809 | lemma set_insert: | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 810 | assumes "x \<in> A" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 811 | obtains B where "A = insert x B" and "x \<notin> B" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 812 | proof | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 813 |   from assms show "A = insert x (A - {x})" by blast
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 814 | next | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 815 |   show "x \<notin> A - {x}" by blast
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 816 | qed | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 817 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 818 | lemma insert_ident: "x ~: A ==> x ~: B ==> (insert x A = insert x B) = (A = B)" | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 819 | by auto | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 820 | |
| 44744 | 821 | lemma insert_eq_iff: assumes "a \<notin> A" "b \<notin> B" | 
| 822 | shows "insert a A = insert b B \<longleftrightarrow> | |
| 823 | (if a=b then A=B else \<exists>C. A = insert b C \<and> b \<notin> C \<and> B = insert a C \<and> a \<notin> C)" | |
| 824 | (is "?L \<longleftrightarrow> ?R") | |
| 825 | proof | |
| 826 | assume ?L | |
| 827 | show ?R | |
| 828 | proof cases | |
| 829 | assume "a=b" with assms `?L` show ?R by (simp add: insert_ident) | |
| 830 | next | |
| 831 | assume "a\<noteq>b" | |
| 832 |     let ?C = "A - {b}"
 | |
| 833 | have "A = insert b ?C \<and> b \<notin> ?C \<and> B = insert a ?C \<and> a \<notin> ?C" | |
| 834 | using assms `?L` `a\<noteq>b` by auto | |
| 835 | thus ?R using `a\<noteq>b` by auto | |
| 836 | qed | |
| 837 | next | |
| 46128 
53e7cc599f58
interaction of set operations for execution and membership predicate
 haftmann parents: 
46127diff
changeset | 838 | assume ?R thus ?L by (auto split: if_splits) | 
| 44744 | 839 | qed | 
| 840 | ||
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 841 | subsubsection {* Singletons, using insert *}
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 842 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 843 | lemma singletonI [intro!,no_atp]: "a : {a}"
 | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 844 |     -- {* Redundant? But unlike @{text insertCI}, it proves the subgoal immediately! *}
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 845 | by (rule insertI1) | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 846 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 847 | lemma singletonD [dest!,no_atp]: "b : {a} ==> b = a"
 | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 848 | by blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 849 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 850 | lemmas singletonE = singletonD [elim_format] | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 851 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 852 | lemma singleton_iff: "(b : {a}) = (b = a)"
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 853 | by blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 854 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 855 | lemma singleton_inject [dest!]: "{a} = {b} ==> a = b"
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 856 | by blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 857 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 858 | lemma singleton_insert_inj_eq [iff,no_atp]: | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 859 |      "({b} = insert a A) = (a = b & A \<subseteq> {b})"
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 860 | by blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 861 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 862 | lemma singleton_insert_inj_eq' [iff,no_atp]: | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 863 |      "(insert a A = {b}) = (a = b & A \<subseteq> {b})"
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 864 | by blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 865 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 866 | lemma subset_singletonD: "A \<subseteq> {x} ==> A = {} | A = {x}"
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 867 | by fast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 868 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 869 | lemma singleton_conv [simp]: "{x. x = a} = {a}"
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 870 | by blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 871 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 872 | lemma singleton_conv2 [simp]: "{x. a = x} = {a}"
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 873 | by blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 874 | |
| 46504 
cd4832aa2229
removing unnecessary premise from diff_single_insert
 bulwahn parents: 
46459diff
changeset | 875 | lemma diff_single_insert: "A - {x} \<subseteq> B ==> A \<subseteq> insert x B"
 | 
| 30531 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 876 | by blast | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 877 | |
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 878 | lemma doubleton_eq_iff: "({a,b} = {c,d}) = (a=c & b=d | a=d & b=c)"
 | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 879 | by (blast elim: equalityE) | 
| 
ab3d61baf66a
reverted to old version of Set.thy -- strange effects have to be traced first
 haftmann parents: 
30352diff
changeset | 880 | |
| 11979 | 881 | |
| 32077 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 882 | subsubsection {* Image of a set under a function *}
 | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 883 | |
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 884 | text {*
 | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 885 |   Frequently @{term b} does not have the syntactic form of @{term "f x"}.
 | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 886 | *} | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 887 | |
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 888 | definition image :: "('a => 'b) => 'a set => 'b set" (infixr "`" 90) where
 | 
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 889 |   image_def [no_atp]: "f ` A = {y. EX x:A. y = f(x)}"
 | 
| 32077 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 890 | |
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 891 | abbreviation | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 892 |   range :: "('a => 'b) => 'b set" where -- "of function"
 | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 893 | "range f == f ` UNIV" | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 894 | |
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 895 | lemma image_eqI [simp, intro]: "b = f x ==> x:A ==> b : f`A" | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 896 | by (unfold image_def) blast | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 897 | |
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 898 | lemma imageI: "x : A ==> f x : f ` A" | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 899 | by (rule image_eqI) (rule refl) | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 900 | |
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 901 | lemma rev_image_eqI: "x:A ==> b = f x ==> b : f`A" | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 902 |   -- {* This version's more effective when we already have the
 | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 903 |     required @{term x}. *}
 | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 904 | by (unfold image_def) blast | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 905 | |
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 906 | lemma imageE [elim!]: | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 907 | "b : (%x. f x)`A ==> (!!x. b = f x ==> x:A ==> P) ==> P" | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 908 |   -- {* The eta-expansion gives variable-name preservation. *}
 | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 909 | by (unfold image_def) blast | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 910 | |
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 911 | lemma image_Un: "f`(A Un B) = f`A Un f`B" | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 912 | by blast | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 913 | |
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 914 | lemma image_iff: "(z : f`A) = (EX x:A. z = f x)" | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 915 | by blast | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 916 | |
| 38648 
52ea97d95e4b
"no_atp" a few facts that often lead to unsound proofs
 blanchet parents: 
37767diff
changeset | 917 | lemma image_subset_iff [no_atp]: "(f`A \<subseteq> B) = (\<forall>x\<in>A. f x \<in> B)" | 
| 32077 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 918 |   -- {* This rewrite rule would confuse users if made default. *}
 | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 919 | by blast | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 920 | |
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 921 | lemma subset_image_iff: "(B \<subseteq> f`A) = (EX AA. AA \<subseteq> A & B = f`AA)" | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 922 | apply safe | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 923 | prefer 2 apply fast | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 924 |   apply (rule_tac x = "{a. a : A & f a : B}" in exI, fast)
 | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 925 | done | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 926 | |
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 927 | lemma image_subsetI: "(!!x. x \<in> A ==> f x \<in> B) ==> f`A \<subseteq> B" | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 928 |   -- {* Replaces the three steps @{text subsetI}, @{text imageE},
 | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 929 |     @{text hypsubst}, but breaks too many existing proofs. *}
 | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 930 | by blast | 
| 11979 | 931 | |
| 932 | text {*
 | |
| 32077 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 933 | \medskip Range of a function -- just a translation for image! | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 934 | *} | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 935 | |
| 43898 | 936 | lemma image_ident [simp]: "(%x. x) ` Y = Y" | 
| 937 | by blast | |
| 938 | ||
| 32077 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 939 | lemma range_eqI: "b = f x ==> b \<in> range f" | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 940 | by simp | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 941 | |
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 942 | lemma rangeI: "f x \<in> range f" | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 943 | by simp | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 944 | |
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 945 | lemma rangeE [elim?]: "b \<in> range (\<lambda>x. f x) ==> (!!x. b = f x ==> P) ==> P" | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 946 | by blast | 
| 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 947 | |
| 32117 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 948 | subsubsection {* Some rules with @{text "if"} *}
 | 
| 32081 | 949 | |
| 950 | text{* Elimination of @{text"{x. \<dots> & x=t & \<dots>}"}. *}
 | |
| 951 | ||
| 952 | lemma Collect_conv_if: "{x. x=a & P x} = (if P a then {a} else {})"
 | |
| 32117 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 953 | by auto | 
| 32081 | 954 | |
| 955 | lemma Collect_conv_if2: "{x. a=x & P x} = (if P a then {a} else {})"
 | |
| 32117 
0762b9ad83df
Set.thy: prefer = over == where possible; tuned ML setup; dropped (moved) ML legacy
 haftmann parents: 
32115diff
changeset | 956 | by auto | 
| 32081 | 957 | |
| 958 | text {*
 | |
| 959 |   Rewrite rules for boolean case-splitting: faster than @{text
 | |
| 960 | "split_if [split]"}. | |
| 961 | *} | |
| 962 | ||
| 963 | lemma split_if_eq1: "((if Q then x else y) = b) = ((Q --> x = b) & (~ Q --> y = b))" | |
| 964 | by (rule split_if) | |
| 965 | ||
| 966 | lemma split_if_eq2: "(a = (if Q then x else y)) = ((Q --> a = x) & (~ Q --> a = y))" | |
| 967 | by (rule split_if) | |
| 968 | ||
| 969 | text {*
 | |
| 970 |   Split ifs on either side of the membership relation.  Not for @{text
 | |
| 971 | "[simp]"} -- can cause goals to blow up! | |
| 972 | *} | |
| 973 | ||
| 974 | lemma split_if_mem1: "((if Q then x else y) : b) = ((Q --> x : b) & (~ Q --> y : b))" | |
| 975 | by (rule split_if) | |
| 976 | ||
| 977 | lemma split_if_mem2: "(a : (if Q then x else y)) = ((Q --> a : x) & (~ Q --> a : y))" | |
| 978 | by (rule split_if [where P="%S. a : S"]) | |
| 979 | ||
| 980 | lemmas split_ifs = if_bool_eq_conj split_if_eq1 split_if_eq2 split_if_mem1 split_if_mem2 | |
| 981 | ||
| 982 | (*Would like to add these, but the existing code only searches for the | |
| 37677 | 983 | outer-level constant, which in this case is just Set.member; we instead need | 
| 32081 | 984 | to use term-nets to associate patterns with rules. Also, if a rule fails to | 
| 985 | apply, then the formula should be kept. | |
| 34974 
18b41bba42b5
new theory Algebras.thy for generic algebraic structures
 haftmann parents: 
34209diff
changeset | 986 |   [("uminus", Compl_iff RS iffD1), ("minus", [Diff_iff RS iffD1]),
 | 
| 32081 | 987 |    ("Int", [IntD1,IntD2]),
 | 
| 988 |    ("Collect", [CollectD]), ("Inter", [InterD]), ("INTER", [INT_D])]
 | |
| 989 | *) | |
| 990 | ||
| 991 | ||
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 992 | subsection {* Further operations and lemmas *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 993 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 994 | subsubsection {* The ``proper subset'' relation *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 995 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 996 | lemma psubsetI [intro!,no_atp]: "A \<subseteq> B ==> A \<noteq> B ==> A \<subset> B" | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 997 | by (unfold less_le) blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 998 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 999 | lemma psubsetE [elim!,no_atp]: | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1000 | "[|A \<subset> B; [|A \<subseteq> B; ~ (B\<subseteq>A)|] ==> R|] ==> R" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1001 | by (unfold less_le) blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1002 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1003 | lemma psubset_insert_iff: | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1004 |   "(A \<subset> insert x B) = (if x \<in> B then A \<subset> B else if x \<in> A then A - {x} \<subset> B else A \<subseteq> B)"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1005 | by (auto simp add: less_le subset_insert_iff) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1006 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1007 | lemma psubset_eq: "(A \<subset> B) = (A \<subseteq> B & A \<noteq> B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1008 | by (simp only: less_le) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1009 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1010 | lemma psubset_imp_subset: "A \<subset> B ==> A \<subseteq> B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1011 | by (simp add: psubset_eq) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1012 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1013 | lemma psubset_trans: "[| A \<subset> B; B \<subset> C |] ==> A \<subset> C" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1014 | apply (unfold less_le) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1015 | apply (auto dest: subset_antisym) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1016 | done | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1017 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1018 | lemma psubsetD: "[| A \<subset> B; c \<in> A |] ==> c \<in> B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1019 | apply (unfold less_le) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1020 | apply (auto dest: subsetD) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1021 | done | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1022 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1023 | lemma psubset_subset_trans: "A \<subset> B ==> B \<subseteq> C ==> A \<subset> C" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1024 | by (auto simp add: psubset_eq) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1025 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1026 | lemma subset_psubset_trans: "A \<subseteq> B ==> B \<subset> C ==> A \<subset> C" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1027 | by (auto simp add: psubset_eq) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1028 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1029 | lemma psubset_imp_ex_mem: "A \<subset> B ==> \<exists>b. b \<in> (B - A)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1030 | by (unfold less_le) blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1031 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1032 | lemma atomize_ball: | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1033 | "(!!x. x \<in> A ==> P x) == Trueprop (\<forall>x\<in>A. P x)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1034 | by (simp only: Ball_def atomize_all atomize_imp) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1035 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1036 | lemmas [symmetric, rulify] = atomize_ball | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1037 | and [symmetric, defn] = atomize_ball | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1038 | |
| 40703 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1039 | lemma image_Pow_mono: | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1040 | assumes "f ` A \<le> B" | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1041 | shows "(image f) ` (Pow A) \<le> Pow B" | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1042 | using assms by blast | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1043 | |
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1044 | lemma image_Pow_surj: | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1045 | assumes "f ` A = B" | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1046 | shows "(image f) ` (Pow A) = Pow B" | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1047 | using assms unfolding Pow_def proof(auto) | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1048 | fix Y assume *: "Y \<le> f ` A" | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1049 |   obtain X where X_def: "X = {x \<in> A. f x \<in> Y}" by blast
 | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1050 | have "f ` X = Y \<and> X \<le> A" unfolding X_def using * by auto | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1051 |   thus "Y \<in> (image f) ` {X. X \<le> A}" by blast
 | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1052 | qed | 
| 
d1fc454d6735
Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
 hoelzl parents: 
39910diff
changeset | 1053 | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1054 | subsubsection {* Derived rules involving subsets. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1055 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1056 | text {* @{text insert}. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1057 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1058 | lemma subset_insertI: "B \<subseteq> insert a B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1059 | by (rule subsetI) (erule insertI2) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1060 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1061 | lemma subset_insertI2: "A \<subseteq> B \<Longrightarrow> A \<subseteq> insert b B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1062 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1063 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1064 | lemma subset_insert: "x \<notin> A ==> (A \<subseteq> insert x B) = (A \<subseteq> B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1065 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1066 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1067 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1068 | text {* \medskip Finite Union -- the least upper bound of two sets. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1069 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1070 | lemma Un_upper1: "A \<subseteq> A \<union> B" | 
| 36009 | 1071 | by (fact sup_ge1) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1072 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1073 | lemma Un_upper2: "B \<subseteq> A \<union> B" | 
| 36009 | 1074 | by (fact sup_ge2) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1075 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1076 | lemma Un_least: "A \<subseteq> C ==> B \<subseteq> C ==> A \<union> B \<subseteq> C" | 
| 36009 | 1077 | by (fact sup_least) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1078 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1079 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1080 | text {* \medskip Finite Intersection -- the greatest lower bound of two sets. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1081 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1082 | lemma Int_lower1: "A \<inter> B \<subseteq> A" | 
| 36009 | 1083 | by (fact inf_le1) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1084 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1085 | lemma Int_lower2: "A \<inter> B \<subseteq> B" | 
| 36009 | 1086 | by (fact inf_le2) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1087 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1088 | lemma Int_greatest: "C \<subseteq> A ==> C \<subseteq> B ==> C \<subseteq> A \<inter> B" | 
| 36009 | 1089 | by (fact inf_greatest) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1090 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1091 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1092 | text {* \medskip Set difference. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1093 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1094 | lemma Diff_subset: "A - B \<subseteq> A" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1095 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1096 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1097 | lemma Diff_subset_conv: "(A - B \<subseteq> C) = (A \<subseteq> B \<union> C)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1098 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1099 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1100 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1101 | subsubsection {* Equalities involving union, intersection, inclusion, etc. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1102 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1103 | text {* @{text "{}"}. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1104 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1105 | lemma Collect_const [simp]: "{s. P} = (if P then UNIV else {})"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1106 |   -- {* supersedes @{text "Collect_False_empty"} *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1107 | by auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1108 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1109 | lemma subset_empty [simp]: "(A \<subseteq> {}) = (A = {})"
 | 
| 45121 | 1110 | by (fact bot_unique) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1111 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1112 | lemma not_psubset_empty [iff]: "\<not> (A < {})"
 | 
| 45121 | 1113 | by (fact not_less_bot) (* FIXME: already simp *) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1114 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1115 | lemma Collect_empty_eq [simp]: "(Collect P = {}) = (\<forall>x. \<not> P x)"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1116 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1117 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1118 | lemma empty_Collect_eq [simp]: "({} = Collect P) = (\<forall>x. \<not> P x)"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1119 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1120 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1121 | lemma Collect_neg_eq: "{x. \<not> P x} = - {x. P x}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1122 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1123 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1124 | lemma Collect_disj_eq: "{x. P x | Q x} = {x. P x} \<union> {x. Q x}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1125 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1126 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1127 | lemma Collect_imp_eq: "{x. P x --> Q x} = -{x. P x} \<union> {x. Q x}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1128 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1129 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1130 | lemma Collect_conj_eq: "{x. P x & Q x} = {x. P x} \<inter> {x. Q x}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1131 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1132 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1133 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1134 | text {* \medskip @{text insert}. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1135 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1136 | lemma insert_is_Un: "insert a A = {a} Un A"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1137 |   -- {* NOT SUITABLE FOR REWRITING since @{text "{a} == insert a {}"} *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1138 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1139 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1140 | lemma insert_not_empty [simp]: "insert a A \<noteq> {}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1141 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1142 | |
| 45607 | 1143 | lemmas empty_not_insert = insert_not_empty [symmetric] | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1144 | declare empty_not_insert [simp] | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1145 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1146 | lemma insert_absorb: "a \<in> A ==> insert a A = A" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1147 |   -- {* @{text "[simp]"} causes recursive calls when there are nested inserts *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1148 |   -- {* with \emph{quadratic} running time *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1149 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1150 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1151 | lemma insert_absorb2 [simp]: "insert x (insert x A) = insert x A" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1152 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1153 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1154 | lemma insert_commute: "insert x (insert y A) = insert y (insert x A)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1155 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1156 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1157 | lemma insert_subset [simp]: "(insert x A \<subseteq> B) = (x \<in> B & A \<subseteq> B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1158 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1159 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1160 | lemma mk_disjoint_insert: "a \<in> A ==> \<exists>B. A = insert a B & a \<notin> B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1161 |   -- {* use new @{text B} rather than @{text "A - {a}"} to avoid infinite unfolding *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1162 |   apply (rule_tac x = "A - {a}" in exI, blast)
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1163 | done | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1164 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1165 | lemma insert_Collect: "insert a (Collect P) = {u. u \<noteq> a --> P u}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1166 | by auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1167 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1168 | lemma insert_inter_insert[simp]: "insert a A \<inter> insert a B = insert a (A \<inter> B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1169 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1170 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 1171 | lemma insert_disjoint [simp,no_atp]: | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1172 |  "(insert a A \<inter> B = {}) = (a \<notin> B \<and> A \<inter> B = {})"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1173 |  "({} = insert a A \<inter> B) = (a \<notin> B \<and> {} = A \<inter> B)"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1174 | by auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1175 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 1176 | lemma disjoint_insert [simp,no_atp]: | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1177 |  "(B \<inter> insert a A = {}) = (a \<notin> B \<and> B \<inter> A = {})"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1178 |  "({} = A \<inter> insert b B) = (b \<notin> A \<and> {} = A \<inter> B)"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1179 | by auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1180 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1181 | text {* \medskip @{text image}. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1182 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1183 | lemma image_empty [simp]: "f`{} = {}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1184 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1185 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1186 | lemma image_insert [simp]: "f ` insert a B = insert (f a) (f`B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1187 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1188 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1189 | lemma image_constant: "x \<in> A ==> (\<lambda>x. c) ` A = {c}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1190 | by auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1191 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1192 | lemma image_constant_conv: "(%x. c) ` A = (if A = {} then {} else {c})"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1193 | by auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1194 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1195 | lemma image_image: "f ` (g ` A) = (\<lambda>x. f (g x)) ` A" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1196 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1197 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1198 | lemma insert_image [simp]: "x \<in> A ==> insert (f x) (f`A) = f`A" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1199 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1200 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1201 | lemma image_is_empty [iff]: "(f`A = {}) = (A = {})"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1202 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1203 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1204 | lemma empty_is_image[iff]: "({} = f ` A) = (A = {})"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1205 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1206 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1207 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 1208 | lemma image_Collect [no_atp]: "f ` {x. P x} = {f x | x. P x}"
 | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1209 |   -- {* NOT suitable as a default simprule: the RHS isn't simpler than the LHS,
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1210 | with its implicit quantifier and conjunction. Also image enjoys better | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1211 | equational properties than does the RHS. *} | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1212 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1213 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1214 | lemma if_image_distrib [simp]: | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1215 | "(\<lambda>x. if P x then f x else g x) ` S | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1216 |     = (f ` (S \<inter> {x. P x})) \<union> (g ` (S \<inter> {x. \<not> P x}))"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1217 | by (auto simp add: image_def) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1218 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1219 | lemma image_cong: "M = N ==> (!!x. x \<in> N ==> f x = g x) ==> f`M = g`N" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1220 | by (simp add: image_def) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1221 | |
| 43898 | 1222 | lemma image_Int_subset: "f`(A Int B) <= f`A Int f`B" | 
| 1223 | by blast | |
| 1224 | ||
| 1225 | lemma image_diff_subset: "f`A - f`B <= f`(A - B)" | |
| 1226 | by blast | |
| 1227 | ||
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1228 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1229 | text {* \medskip @{text range}. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1230 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 1231 | lemma full_SetCompr_eq [no_atp]: "{u. \<exists>x. u = f x} = range f"
 | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1232 | by auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1233 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1234 | lemma range_composition: "range (\<lambda>x. f (g x)) = f`range g" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1235 | by (subst image_image, simp) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1236 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1237 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1238 | text {* \medskip @{text Int} *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1239 | |
| 45121 | 1240 | lemma Int_absorb: "A \<inter> A = A" | 
| 1241 | by (fact inf_idem) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1242 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1243 | lemma Int_left_absorb: "A \<inter> (A \<inter> B) = A \<inter> B" | 
| 36009 | 1244 | by (fact inf_left_idem) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1245 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1246 | lemma Int_commute: "A \<inter> B = B \<inter> A" | 
| 36009 | 1247 | by (fact inf_commute) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1248 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1249 | lemma Int_left_commute: "A \<inter> (B \<inter> C) = B \<inter> (A \<inter> C)" | 
| 36009 | 1250 | by (fact inf_left_commute) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1251 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1252 | lemma Int_assoc: "(A \<inter> B) \<inter> C = A \<inter> (B \<inter> C)" | 
| 36009 | 1253 | by (fact inf_assoc) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1254 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1255 | lemmas Int_ac = Int_assoc Int_left_absorb Int_commute Int_left_commute | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1256 |   -- {* Intersection is an AC-operator *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1257 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1258 | lemma Int_absorb1: "B \<subseteq> A ==> A \<inter> B = B" | 
| 36009 | 1259 | by (fact inf_absorb2) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1260 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1261 | lemma Int_absorb2: "A \<subseteq> B ==> A \<inter> B = A" | 
| 36009 | 1262 | by (fact inf_absorb1) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1263 | |
| 45121 | 1264 | lemma Int_empty_left: "{} \<inter> B = {}"
 | 
| 1265 | by (fact inf_bot_left) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1266 | |
| 45121 | 1267 | lemma Int_empty_right: "A \<inter> {} = {}"
 | 
| 1268 | by (fact inf_bot_right) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1269 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1270 | lemma disjoint_eq_subset_Compl: "(A \<inter> B = {}) = (A \<subseteq> -B)"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1271 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1272 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1273 | lemma disjoint_iff_not_equal: "(A \<inter> B = {}) = (\<forall>x\<in>A. \<forall>y\<in>B. x \<noteq> y)"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1274 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1275 | |
| 45121 | 1276 | lemma Int_UNIV_left: "UNIV \<inter> B = B" | 
| 1277 | by (fact inf_top_left) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1278 | |
| 45121 | 1279 | lemma Int_UNIV_right: "A \<inter> UNIV = A" | 
| 1280 | by (fact inf_top_right) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1281 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1282 | lemma Int_Un_distrib: "A \<inter> (B \<union> C) = (A \<inter> B) \<union> (A \<inter> C)" | 
| 36009 | 1283 | by (fact inf_sup_distrib1) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1284 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1285 | lemma Int_Un_distrib2: "(B \<union> C) \<inter> A = (B \<inter> A) \<union> (C \<inter> A)" | 
| 36009 | 1286 | by (fact inf_sup_distrib2) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1287 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 1288 | lemma Int_UNIV [simp,no_atp]: "(A \<inter> B = UNIV) = (A = UNIV & B = UNIV)" | 
| 45121 | 1289 | by (fact inf_eq_top_iff) (* already simp *) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1290 | |
| 38648 
52ea97d95e4b
"no_atp" a few facts that often lead to unsound proofs
 blanchet parents: 
37767diff
changeset | 1291 | lemma Int_subset_iff [no_atp, simp]: "(C \<subseteq> A \<inter> B) = (C \<subseteq> A & C \<subseteq> B)" | 
| 36009 | 1292 | by (fact le_inf_iff) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1293 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1294 | lemma Int_Collect: "(x \<in> A \<inter> {x. P x}) = (x \<in> A & P x)"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1295 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1296 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1297 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1298 | text {* \medskip @{text Un}. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1299 | |
| 45121 | 1300 | lemma Un_absorb: "A \<union> A = A" | 
| 1301 | by (fact sup_idem) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1302 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1303 | lemma Un_left_absorb: "A \<union> (A \<union> B) = A \<union> B" | 
| 36009 | 1304 | by (fact sup_left_idem) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1305 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1306 | lemma Un_commute: "A \<union> B = B \<union> A" | 
| 36009 | 1307 | by (fact sup_commute) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1308 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1309 | lemma Un_left_commute: "A \<union> (B \<union> C) = B \<union> (A \<union> C)" | 
| 36009 | 1310 | by (fact sup_left_commute) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1311 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1312 | lemma Un_assoc: "(A \<union> B) \<union> C = A \<union> (B \<union> C)" | 
| 36009 | 1313 | by (fact sup_assoc) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1314 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1315 | lemmas Un_ac = Un_assoc Un_left_absorb Un_commute Un_left_commute | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1316 |   -- {* Union is an AC-operator *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1317 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1318 | lemma Un_absorb1: "A \<subseteq> B ==> A \<union> B = B" | 
| 36009 | 1319 | by (fact sup_absorb2) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1320 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1321 | lemma Un_absorb2: "B \<subseteq> A ==> A \<union> B = A" | 
| 36009 | 1322 | by (fact sup_absorb1) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1323 | |
| 45121 | 1324 | lemma Un_empty_left: "{} \<union> B = B"
 | 
| 1325 | by (fact sup_bot_left) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1326 | |
| 45121 | 1327 | lemma Un_empty_right: "A \<union> {} = A"
 | 
| 1328 | by (fact sup_bot_right) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1329 | |
| 45121 | 1330 | lemma Un_UNIV_left: "UNIV \<union> B = UNIV" | 
| 1331 | by (fact sup_top_left) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1332 | |
| 45121 | 1333 | lemma Un_UNIV_right: "A \<union> UNIV = UNIV" | 
| 1334 | by (fact sup_top_right) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1335 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1336 | lemma Un_insert_left [simp]: "(insert a B) \<union> C = insert a (B \<union> C)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1337 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1338 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1339 | lemma Un_insert_right [simp]: "A \<union> (insert a B) = insert a (A \<union> B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1340 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1341 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1342 | lemma Int_insert_left: | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1343 | "(insert a B) Int C = (if a \<in> C then insert a (B \<inter> C) else B \<inter> C)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1344 | by auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1345 | |
| 32456 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1346 | lemma Int_insert_left_if0[simp]: | 
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1347 | "a \<notin> C \<Longrightarrow> (insert a B) Int C = B \<inter> C" | 
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1348 | by auto | 
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1349 | |
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1350 | lemma Int_insert_left_if1[simp]: | 
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1351 | "a \<in> C \<Longrightarrow> (insert a B) Int C = insert a (B Int C)" | 
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1352 | by auto | 
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1353 | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1354 | lemma Int_insert_right: | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1355 | "A \<inter> (insert a B) = (if a \<in> A then insert a (A \<inter> B) else A \<inter> B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1356 | by auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1357 | |
| 32456 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1358 | lemma Int_insert_right_if0[simp]: | 
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1359 | "a \<notin> A \<Longrightarrow> A Int (insert a B) = A Int B" | 
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1360 | by auto | 
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1361 | |
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1362 | lemma Int_insert_right_if1[simp]: | 
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1363 | "a \<in> A \<Longrightarrow> A Int (insert a B) = insert a (A Int B)" | 
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1364 | by auto | 
| 
341c83339aeb
tuned the simp rules for Int involving insert and intervals.
 nipkow parents: 
32264diff
changeset | 1365 | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1366 | lemma Un_Int_distrib: "A \<union> (B \<inter> C) = (A \<union> B) \<inter> (A \<union> C)" | 
| 36009 | 1367 | by (fact sup_inf_distrib1) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1368 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1369 | lemma Un_Int_distrib2: "(B \<inter> C) \<union> A = (B \<union> A) \<inter> (C \<union> A)" | 
| 36009 | 1370 | by (fact sup_inf_distrib2) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1371 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1372 | lemma Un_Int_crazy: | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1373 | "(A \<inter> B) \<union> (B \<inter> C) \<union> (C \<inter> A) = (A \<union> B) \<inter> (B \<union> C) \<inter> (C \<union> A)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1374 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1375 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1376 | lemma subset_Un_eq: "(A \<subseteq> B) = (A \<union> B = B)" | 
| 36009 | 1377 | by (fact le_iff_sup) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1378 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1379 | lemma Un_empty [iff]: "(A \<union> B = {}) = (A = {} & B = {})"
 | 
| 45121 | 1380 | by (fact sup_eq_bot_iff) (* FIXME: already simp *) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1381 | |
| 38648 
52ea97d95e4b
"no_atp" a few facts that often lead to unsound proofs
 blanchet parents: 
37767diff
changeset | 1382 | lemma Un_subset_iff [no_atp, simp]: "(A \<union> B \<subseteq> C) = (A \<subseteq> C & B \<subseteq> C)" | 
| 36009 | 1383 | by (fact le_sup_iff) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1384 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1385 | lemma Un_Diff_Int: "(A - B) \<union> (A \<inter> B) = A" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1386 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1387 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1388 | lemma Diff_Int2: "A \<inter> C - B \<inter> C = A \<inter> C - B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1389 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1390 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1391 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1392 | text {* \medskip Set complement *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1393 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1394 | lemma Compl_disjoint [simp]: "A \<inter> -A = {}"
 | 
| 36009 | 1395 | by (fact inf_compl_bot) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1396 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1397 | lemma Compl_disjoint2 [simp]: "-A \<inter> A = {}"
 | 
| 36009 | 1398 | by (fact compl_inf_bot) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1399 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1400 | lemma Compl_partition: "A \<union> -A = UNIV" | 
| 36009 | 1401 | by (fact sup_compl_top) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1402 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1403 | lemma Compl_partition2: "-A \<union> A = UNIV" | 
| 36009 | 1404 | by (fact compl_sup_top) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1405 | |
| 45121 | 1406 | lemma double_complement: "- (-A) = (A::'a set)" | 
| 1407 | by (fact double_compl) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1408 | |
| 45121 | 1409 | lemma Compl_Un: "-(A \<union> B) = (-A) \<inter> (-B)" | 
| 1410 | by (fact compl_sup) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1411 | |
| 45121 | 1412 | lemma Compl_Int: "-(A \<inter> B) = (-A) \<union> (-B)" | 
| 1413 | by (fact compl_inf) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1414 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1415 | lemma subset_Compl_self_eq: "(A \<subseteq> -A) = (A = {})"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1416 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1417 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1418 | lemma Un_Int_assoc_eq: "((A \<inter> B) \<union> C = A \<inter> (B \<union> C)) = (C \<subseteq> A)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1419 |   -- {* Halmos, Naive Set Theory, page 16. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1420 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1421 | |
| 45121 | 1422 | lemma Compl_UNIV_eq: "-UNIV = {}"
 | 
| 1423 | by (fact compl_top_eq) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1424 | |
| 45121 | 1425 | lemma Compl_empty_eq: "-{} = UNIV"
 | 
| 1426 | by (fact compl_bot_eq) (* already simp *) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1427 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1428 | lemma Compl_subset_Compl_iff [iff]: "(-A \<subseteq> -B) = (B \<subseteq> A)" | 
| 45121 | 1429 | by (fact compl_le_compl_iff) (* FIXME: already simp *) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1430 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1431 | lemma Compl_eq_Compl_iff [iff]: "(-A = -B) = (A = (B::'a set))" | 
| 45121 | 1432 | by (fact compl_eq_compl_iff) (* FIXME: already simp *) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1433 | |
| 44490 | 1434 | lemma Compl_insert: "- insert x A = (-A) - {x}"
 | 
| 1435 | by blast | |
| 1436 | ||
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1437 | text {* \medskip Bounded quantifiers.
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1438 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1439 | The following are not added to the default simpset because | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1440 |   (a) they duplicate the body and (b) there are no similar rules for @{text Int}. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1441 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1442 | lemma ball_Un: "(\<forall>x \<in> A \<union> B. P x) = ((\<forall>x\<in>A. P x) & (\<forall>x\<in>B. P x))" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1443 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1444 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1445 | lemma bex_Un: "(\<exists>x \<in> A \<union> B. P x) = ((\<exists>x\<in>A. P x) | (\<exists>x\<in>B. P x))" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1446 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1447 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1448 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1449 | text {* \medskip Set difference. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1450 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1451 | lemma Diff_eq: "A - B = A \<inter> (-B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1452 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1453 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 1454 | lemma Diff_eq_empty_iff [simp,no_atp]: "(A - B = {}) = (A \<subseteq> B)"
 | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1455 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1456 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1457 | lemma Diff_cancel [simp]: "A - A = {}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1458 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1459 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1460 | lemma Diff_idemp [simp]: "(A - B) - B = A - (B::'a set)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1461 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1462 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1463 | lemma Diff_triv: "A \<inter> B = {} ==> A - B = A"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1464 | by (blast elim: equalityE) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1465 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1466 | lemma empty_Diff [simp]: "{} - A = {}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1467 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1468 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1469 | lemma Diff_empty [simp]: "A - {} = A"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1470 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1471 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1472 | lemma Diff_UNIV [simp]: "A - UNIV = {}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1473 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1474 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 1475 | lemma Diff_insert0 [simp,no_atp]: "x \<notin> A ==> A - insert x B = A - B" | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1476 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1477 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1478 | lemma Diff_insert: "A - insert a B = A - B - {a}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1479 |   -- {* NOT SUITABLE FOR REWRITING since @{text "{a} == insert a 0"} *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1480 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1481 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1482 | lemma Diff_insert2: "A - insert a B = A - {a} - B"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1483 |   -- {* NOT SUITABLE FOR REWRITING since @{text "{a} == insert a 0"} *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1484 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1485 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1486 | lemma insert_Diff_if: "insert x A - B = (if x \<in> B then A - B else insert x (A - B))" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1487 | by auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1488 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1489 | lemma insert_Diff1 [simp]: "x \<in> B ==> insert x A - B = A - B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1490 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1491 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1492 | lemma insert_Diff_single[simp]: "insert a (A - {a}) = insert a A"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1493 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1494 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1495 | lemma insert_Diff: "a \<in> A ==> insert a (A - {a}) = A"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1496 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1497 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1498 | lemma Diff_insert_absorb: "x \<notin> A ==> (insert x A) - {x} = A"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1499 | by auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1500 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1501 | lemma Diff_disjoint [simp]: "A \<inter> (B - A) = {}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1502 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1503 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1504 | lemma Diff_partition: "A \<subseteq> B ==> A \<union> (B - A) = B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1505 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1506 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1507 | lemma double_diff: "A \<subseteq> B ==> B \<subseteq> C ==> B - (C - A) = A" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1508 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1509 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1510 | lemma Un_Diff_cancel [simp]: "A \<union> (B - A) = A \<union> B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1511 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1512 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1513 | lemma Un_Diff_cancel2 [simp]: "(B - A) \<union> A = B \<union> A" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1514 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1515 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1516 | lemma Diff_Un: "A - (B \<union> C) = (A - B) \<inter> (A - C)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1517 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1518 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1519 | lemma Diff_Int: "A - (B \<inter> C) = (A - B) \<union> (A - C)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1520 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1521 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1522 | lemma Un_Diff: "(A \<union> B) - C = (A - C) \<union> (B - C)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1523 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1524 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1525 | lemma Int_Diff: "(A \<inter> B) - C = A \<inter> (B - C)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1526 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1527 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1528 | lemma Diff_Int_distrib: "C \<inter> (A - B) = (C \<inter> A) - (C \<inter> B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1529 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1530 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1531 | lemma Diff_Int_distrib2: "(A - B) \<inter> C = (A \<inter> C) - (B \<inter> C)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1532 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1533 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1534 | lemma Diff_Compl [simp]: "A - (- B) = A \<inter> B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1535 | by auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1536 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1537 | lemma Compl_Diff_eq [simp]: "- (A - B) = -A \<union> B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1538 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1539 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1540 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1541 | text {* \medskip Quantification over type @{typ bool}. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1542 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1543 | lemma bool_induct: "P True \<Longrightarrow> P False \<Longrightarrow> P x" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1544 | by (cases x) auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1545 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1546 | lemma all_bool_eq: "(\<forall>b. P b) \<longleftrightarrow> P True \<and> P False" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1547 | by (auto intro: bool_induct) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1548 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1549 | lemma bool_contrapos: "P x \<Longrightarrow> \<not> P False \<Longrightarrow> P True" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1550 | by (cases x) auto | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1551 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1552 | lemma ex_bool_eq: "(\<exists>b. P b) \<longleftrightarrow> P True \<or> P False" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1553 | by (auto intro: bool_contrapos) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1554 | |
| 43866 
8a50dc70cbff
moving UNIV = ... equations to their proper theories
 haftmann parents: 
43818diff
changeset | 1555 | lemma UNIV_bool [no_atp]: "UNIV = {False, True}"
 | 
| 
8a50dc70cbff
moving UNIV = ... equations to their proper theories
 haftmann parents: 
43818diff
changeset | 1556 | by (auto intro: bool_induct) | 
| 
8a50dc70cbff
moving UNIV = ... equations to their proper theories
 haftmann parents: 
43818diff
changeset | 1557 | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1558 | text {* \medskip @{text Pow} *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1559 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1560 | lemma Pow_empty [simp]: "Pow {} = {{}}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1561 | by (auto simp add: Pow_def) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1562 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1563 | lemma Pow_insert: "Pow (insert a A) = Pow A \<union> (insert a ` Pow A)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1564 |   by (blast intro: image_eqI [where ?x = "u - {a}", standard])
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1565 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1566 | lemma Pow_Compl: "Pow (- A) = {-B | B. A \<in> Pow B}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1567 | by (blast intro: exI [where ?x = "- u", standard]) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1568 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1569 | lemma Pow_UNIV [simp]: "Pow UNIV = UNIV" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1570 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1571 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1572 | lemma Un_Pow_subset: "Pow A \<union> Pow B \<subseteq> Pow (A \<union> B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1573 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1574 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1575 | lemma Pow_Int_eq [simp]: "Pow (A \<inter> B) = Pow A \<inter> Pow B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1576 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1577 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1578 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1579 | text {* \medskip Miscellany. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1580 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1581 | lemma set_eq_subset: "(A = B) = (A \<subseteq> B & B \<subseteq> A)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1582 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1583 | |
| 38648 
52ea97d95e4b
"no_atp" a few facts that often lead to unsound proofs
 blanchet parents: 
37767diff
changeset | 1584 | lemma subset_iff [no_atp]: "(A \<subseteq> B) = (\<forall>t. t \<in> A --> t \<in> B)" | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1585 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1586 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1587 | lemma subset_iff_psubset_eq: "(A \<subseteq> B) = ((A \<subset> B) | (A = B))" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1588 | by (unfold less_le) blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1589 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1590 | lemma all_not_in_conv [simp]: "(\<forall>x. x \<notin> A) = (A = {})"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1591 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1592 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1593 | lemma ex_in_conv: "(\<exists>x. x \<in> A) = (A \<noteq> {})"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1594 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1595 | |
| 43967 | 1596 | lemma ball_simps [simp, no_atp]: | 
| 1597 | "\<And>A P Q. (\<forall>x\<in>A. P x \<or> Q) \<longleftrightarrow> ((\<forall>x\<in>A. P x) \<or> Q)" | |
| 1598 | "\<And>A P Q. (\<forall>x\<in>A. P \<or> Q x) \<longleftrightarrow> (P \<or> (\<forall>x\<in>A. Q x))" | |
| 1599 | "\<And>A P Q. (\<forall>x\<in>A. P \<longrightarrow> Q x) \<longleftrightarrow> (P \<longrightarrow> (\<forall>x\<in>A. Q x))" | |
| 1600 | "\<And>A P Q. (\<forall>x\<in>A. P x \<longrightarrow> Q) \<longleftrightarrow> ((\<exists>x\<in>A. P x) \<longrightarrow> Q)" | |
| 1601 |   "\<And>P. (\<forall>x\<in>{}. P x) \<longleftrightarrow> True"
 | |
| 1602 | "\<And>P. (\<forall>x\<in>UNIV. P x) \<longleftrightarrow> (\<forall>x. P x)" | |
| 1603 | "\<And>a B P. (\<forall>x\<in>insert a B. P x) \<longleftrightarrow> (P a \<and> (\<forall>x\<in>B. P x))" | |
| 1604 | "\<And>P Q. (\<forall>x\<in>Collect Q. P x) \<longleftrightarrow> (\<forall>x. Q x \<longrightarrow> P x)" | |
| 1605 | "\<And>A P f. (\<forall>x\<in>f`A. P x) \<longleftrightarrow> (\<forall>x\<in>A. P (f x))" | |
| 1606 | "\<And>A P. (\<not> (\<forall>x\<in>A. P x)) \<longleftrightarrow> (\<exists>x\<in>A. \<not> P x)" | |
| 1607 | by auto | |
| 1608 | ||
| 1609 | lemma bex_simps [simp, no_atp]: | |
| 1610 | "\<And>A P Q. (\<exists>x\<in>A. P x \<and> Q) \<longleftrightarrow> ((\<exists>x\<in>A. P x) \<and> Q)" | |
| 1611 | "\<And>A P Q. (\<exists>x\<in>A. P \<and> Q x) \<longleftrightarrow> (P \<and> (\<exists>x\<in>A. Q x))" | |
| 1612 |   "\<And>P. (\<exists>x\<in>{}. P x) \<longleftrightarrow> False"
 | |
| 1613 | "\<And>P. (\<exists>x\<in>UNIV. P x) \<longleftrightarrow> (\<exists>x. P x)" | |
| 1614 | "\<And>a B P. (\<exists>x\<in>insert a B. P x) \<longleftrightarrow> (P a | (\<exists>x\<in>B. P x))" | |
| 1615 | "\<And>P Q. (\<exists>x\<in>Collect Q. P x) \<longleftrightarrow> (\<exists>x. Q x \<and> P x)" | |
| 1616 | "\<And>A P f. (\<exists>x\<in>f`A. P x) \<longleftrightarrow> (\<exists>x\<in>A. P (f x))" | |
| 1617 | "\<And>A P. (\<not>(\<exists>x\<in>A. P x)) \<longleftrightarrow> (\<forall>x\<in>A. \<not> P x)" | |
| 1618 | by auto | |
| 1619 | ||
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1620 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1621 | subsubsection {* Monotonicity of various operations *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1622 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1623 | lemma image_mono: "A \<subseteq> B ==> f`A \<subseteq> f`B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1624 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1625 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1626 | lemma Pow_mono: "A \<subseteq> B ==> Pow A \<subseteq> Pow B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1627 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1628 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1629 | lemma insert_mono: "C \<subseteq> D ==> insert a C \<subseteq> insert a D" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1630 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1631 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1632 | lemma Un_mono: "A \<subseteq> C ==> B \<subseteq> D ==> A \<union> B \<subseteq> C \<union> D" | 
| 36009 | 1633 | by (fact sup_mono) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1634 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1635 | lemma Int_mono: "A \<subseteq> C ==> B \<subseteq> D ==> A \<inter> B \<subseteq> C \<inter> D" | 
| 36009 | 1636 | by (fact inf_mono) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1637 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1638 | lemma Diff_mono: "A \<subseteq> C ==> D \<subseteq> B ==> A - B \<subseteq> C - D" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1639 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1640 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1641 | lemma Compl_anti_mono: "A \<subseteq> B ==> -B \<subseteq> -A" | 
| 36009 | 1642 | by (fact compl_mono) | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1643 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1644 | text {* \medskip Monotonicity of implications. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1645 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1646 | lemma in_mono: "A \<subseteq> B ==> x \<in> A --> x \<in> B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1647 | apply (rule impI) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1648 | apply (erule subsetD, assumption) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1649 | done | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1650 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1651 | lemma conj_mono: "P1 --> Q1 ==> P2 --> Q2 ==> (P1 & P2) --> (Q1 & Q2)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1652 | by iprover | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1653 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1654 | lemma disj_mono: "P1 --> Q1 ==> P2 --> Q2 ==> (P1 | P2) --> (Q1 | Q2)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1655 | by iprover | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1656 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1657 | lemma imp_mono: "Q1 --> P1 ==> P2 --> Q2 ==> (P1 --> P2) --> (Q1 --> Q2)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1658 | by iprover | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1659 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1660 | lemma imp_refl: "P --> P" .. | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1661 | |
| 33935 | 1662 | lemma not_mono: "Q --> P ==> ~ P --> ~ Q" | 
| 1663 | by iprover | |
| 1664 | ||
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1665 | lemma ex_mono: "(!!x. P x --> Q x) ==> (EX x. P x) --> (EX x. Q x)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1666 | by iprover | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1667 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1668 | lemma all_mono: "(!!x. P x --> Q x) ==> (ALL x. P x) --> (ALL x. Q x)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1669 | by iprover | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1670 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1671 | lemma Collect_mono: "(!!x. P x --> Q x) ==> Collect P \<subseteq> Collect Q" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1672 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1673 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1674 | lemma Int_Collect_mono: | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1675 | "A \<subseteq> B ==> (!!x. x \<in> A ==> P x --> Q x) ==> A \<inter> Collect P \<subseteq> B \<inter> Collect Q" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1676 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1677 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1678 | lemmas basic_monos = | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1679 | subset_refl imp_refl disj_mono conj_mono | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1680 | ex_mono Collect_mono in_mono | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1681 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1682 | lemma eq_to_mono: "a = b ==> c = d ==> b --> d ==> a --> c" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1683 | by iprover | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1684 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1685 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1686 | subsubsection {* Inverse image of a function *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1687 | |
| 35416 
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
 haftmann parents: 
35115diff
changeset | 1688 | definition vimage :: "('a => 'b) => 'b set => 'a set" (infixr "-`" 90) where
 | 
| 37767 | 1689 |   "f -` B == {x. f x : B}"
 | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1690 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1691 | lemma vimage_eq [simp]: "(a : f -` B) = (f a : B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1692 | by (unfold vimage_def) blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1693 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1694 | lemma vimage_singleton_eq: "(a : f -` {b}) = (f a = b)"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1695 | by simp | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1696 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1697 | lemma vimageI [intro]: "f a = b ==> b:B ==> a : f -` B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1698 | by (unfold vimage_def) blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1699 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1700 | lemma vimageI2: "f a : A ==> a : f -` A" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1701 | by (unfold vimage_def) fast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1702 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1703 | lemma vimageE [elim!]: "a: f -` B ==> (!!x. f a = x ==> x:B ==> P) ==> P" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1704 | by (unfold vimage_def) blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1705 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1706 | lemma vimageD: "a : f -` A ==> f a : A" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1707 | by (unfold vimage_def) fast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1708 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1709 | lemma vimage_empty [simp]: "f -` {} = {}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1710 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1711 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1712 | lemma vimage_Compl: "f -` (-A) = -(f -` A)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1713 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1714 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1715 | lemma vimage_Un [simp]: "f -` (A Un B) = (f -` A) Un (f -` B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1716 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1717 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1718 | lemma vimage_Int [simp]: "f -` (A Int B) = (f -` A) Int (f -` B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1719 | by fast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1720 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1721 | lemma vimage_Collect_eq [simp]: "f -` Collect P = {y. P (f y)}"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1722 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1723 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1724 | lemma vimage_Collect: "(!!x. P (f x) = Q x) ==> f -` (Collect P) = Collect Q" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1725 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1726 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1727 | lemma vimage_insert: "f-`(insert a B) = (f-`{a}) Un (f-`B)"
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1728 |   -- {* NOT suitable for rewriting because of the recurrence of @{term "{a}"}. *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1729 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1730 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1731 | lemma vimage_Diff: "f -` (A - B) = (f -` A) - (f -` B)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1732 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1733 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1734 | lemma vimage_UNIV [simp]: "f -` UNIV = UNIV" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1735 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1736 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1737 | lemma vimage_mono: "A \<subseteq> B ==> f -` A \<subseteq> f -` B" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1738 |   -- {* monotonicity *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1739 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1740 | |
| 35828 
46cfc4b8112e
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
 blanchet parents: 
35576diff
changeset | 1741 | lemma vimage_image_eq [no_atp]: "f -` (f ` A) = {y. EX x:A. f x = f y}"
 | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1742 | by (blast intro: sym) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1743 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1744 | lemma image_vimage_subset: "f ` (f -` A) <= A" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1745 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1746 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1747 | lemma image_vimage_eq [simp]: "f ` (f -` A) = A Int range f" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1748 | by blast | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1749 | |
| 33533 
40b44cb20c8c
New theory Probability/Borel.thy, and some associated lemmas
 paulson parents: 
33045diff
changeset | 1750 | lemma vimage_const [simp]: "((\<lambda>x. c) -` A) = (if c \<in> A then UNIV else {})"
 | 
| 
40b44cb20c8c
New theory Probability/Borel.thy, and some associated lemmas
 paulson parents: 
33045diff
changeset | 1751 | by auto | 
| 
40b44cb20c8c
New theory Probability/Borel.thy, and some associated lemmas
 paulson parents: 
33045diff
changeset | 1752 | |
| 
40b44cb20c8c
New theory Probability/Borel.thy, and some associated lemmas
 paulson parents: 
33045diff
changeset | 1753 | lemma vimage_if [simp]: "((\<lambda>x. if x \<in> B then c else d) -` A) = | 
| 
40b44cb20c8c
New theory Probability/Borel.thy, and some associated lemmas
 paulson parents: 
33045diff
changeset | 1754 | (if c \<in> A then (if d \<in> A then UNIV else B) | 
| 
40b44cb20c8c
New theory Probability/Borel.thy, and some associated lemmas
 paulson parents: 
33045diff
changeset | 1755 |     else if d \<in> A then -B else {})"  
 | 
| 
40b44cb20c8c
New theory Probability/Borel.thy, and some associated lemmas
 paulson parents: 
33045diff
changeset | 1756 | by (auto simp add: vimage_def) | 
| 
40b44cb20c8c
New theory Probability/Borel.thy, and some associated lemmas
 paulson parents: 
33045diff
changeset | 1757 | |
| 35576 | 1758 | lemma vimage_inter_cong: | 
| 1759 | "(\<And> w. w \<in> S \<Longrightarrow> f w = g w) \<Longrightarrow> f -` y \<inter> S = g -` y \<inter> S" | |
| 1760 | by auto | |
| 1761 | ||
| 43898 | 1762 | lemma vimage_ident [simp]: "(%x. x) -` Y = Y" | 
| 1763 | by blast | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1764 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1765 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1766 | subsubsection {* Getting the Contents of a Singleton Set *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1767 | |
| 39910 | 1768 | definition the_elem :: "'a set \<Rightarrow> 'a" where | 
| 1769 |   "the_elem X = (THE x. X = {x})"
 | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1770 | |
| 39910 | 1771 | lemma the_elem_eq [simp]: "the_elem {x} = x"
 | 
| 1772 | by (simp add: the_elem_def) | |
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1773 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1774 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1775 | subsubsection {* Least value operator *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1776 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1777 | lemma Least_mono: | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1778 | "mono (f::'a::order => 'b::order) ==> EX x:S. ALL y:S. x <= y | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1779 | ==> (LEAST y. y : f ` S) = f (LEAST x. x : S)" | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1780 |     -- {* Courtesy of Stephan Merz *}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1781 | apply clarify | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1782 | apply (erule_tac P = "%x. x : S" in LeastI2_order, fast) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1783 | apply (rule LeastI2_order) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1784 | apply (auto elim: monoD intro!: order_antisym) | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1785 | done | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1786 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1787 | |
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 1788 | subsubsection {* Monad operation *}
 | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1789 | |
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 1790 | definition bind :: "'a set \<Rightarrow> ('a \<Rightarrow> 'b set) \<Rightarrow> 'b set" where
 | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 1791 |   "bind A f = {x. \<exists>B \<in> f`A. x \<in> B}"
 | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1792 | |
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 1793 | hide_const (open) bind | 
| 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 1794 | |
| 46036 | 1795 | lemma bind_bind: | 
| 1796 | fixes A :: "'a set" | |
| 1797 | shows "Set.bind (Set.bind A B) C = Set.bind A (\<lambda>x. Set.bind (B x) C)" | |
| 1798 | by (auto simp add: bind_def) | |
| 1799 | ||
| 1800 | lemma empty_bind [simp]: | |
| 46128 
53e7cc599f58
interaction of set operations for execution and membership predicate
 haftmann parents: 
46127diff
changeset | 1801 |   "Set.bind {} f = {}"
 | 
| 46036 | 1802 | by (simp add: bind_def) | 
| 1803 | ||
| 1804 | lemma nonempty_bind_const: | |
| 1805 |   "A \<noteq> {} \<Longrightarrow> Set.bind A (\<lambda>_. B) = B"
 | |
| 1806 | by (auto simp add: bind_def) | |
| 1807 | ||
| 1808 | lemma bind_const: "Set.bind A (\<lambda>_. B) = (if A = {} then {} else B)"
 | |
| 1809 | by (auto simp add: bind_def) | |
| 1810 | ||
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 1811 | |
| 45986 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1812 | subsubsection {* Operations for execution *}
 | 
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1813 | |
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1814 | definition is_empty :: "'a set \<Rightarrow> bool" where | 
| 46127 | 1815 |   [code_abbrev]: "is_empty A \<longleftrightarrow> A = {}"
 | 
| 45986 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1816 | |
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1817 | hide_const (open) is_empty | 
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1818 | |
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1819 | definition remove :: "'a \<Rightarrow> 'a set \<Rightarrow> 'a set" where | 
| 46127 | 1820 |   [code_abbrev]: "remove x A = A - {x}"
 | 
| 45986 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1821 | |
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1822 | hide_const (open) remove | 
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1823 | |
| 46128 
53e7cc599f58
interaction of set operations for execution and membership predicate
 haftmann parents: 
46127diff
changeset | 1824 | lemma member_remove [simp]: | 
| 
53e7cc599f58
interaction of set operations for execution and membership predicate
 haftmann parents: 
46127diff
changeset | 1825 | "x \<in> Set.remove y A \<longleftrightarrow> x \<in> A \<and> x \<noteq> y" | 
| 
53e7cc599f58
interaction of set operations for execution and membership predicate
 haftmann parents: 
46127diff
changeset | 1826 | by (simp add: remove_def) | 
| 
53e7cc599f58
interaction of set operations for execution and membership predicate
 haftmann parents: 
46127diff
changeset | 1827 | |
| 45986 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1828 | definition project :: "('a \<Rightarrow> bool) \<Rightarrow> 'a set \<Rightarrow> 'a set" where
 | 
| 46026 
83caa4f4bd56
semiring_numeral_0_eq_0, semiring_numeral_1_eq_1 now [simp], superseeding corresponding simp rules on type nat
 haftmann parents: 
45986diff
changeset | 1829 |   [code_abbrev]: "project P A = {a \<in> A. P a}"
 | 
| 45986 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1830 | |
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1831 | hide_const (open) project | 
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1832 | |
| 46128 
53e7cc599f58
interaction of set operations for execution and membership predicate
 haftmann parents: 
46127diff
changeset | 1833 | lemma member_project [simp]: | 
| 
53e7cc599f58
interaction of set operations for execution and membership predicate
 haftmann parents: 
46127diff
changeset | 1834 | "x \<in> Set.project P A \<longleftrightarrow> x \<in> A \<and> P x" | 
| 
53e7cc599f58
interaction of set operations for execution and membership predicate
 haftmann parents: 
46127diff
changeset | 1835 | by (simp add: project_def) | 
| 
53e7cc599f58
interaction of set operations for execution and membership predicate
 haftmann parents: 
46127diff
changeset | 1836 | |
| 45986 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1837 | instantiation set :: (equal) equal | 
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1838 | begin | 
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1839 | |
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1840 | definition | 
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1841 | "HOL.equal A B \<longleftrightarrow> A \<subseteq> B \<and> B \<subseteq> A" | 
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1842 | |
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1843 | instance proof | 
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1844 | qed (auto simp add: equal_set_def) | 
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1845 | |
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1846 | end | 
| 
c9e50153e5ae
moved various set operations to theory Set (resp. Product_Type)
 haftmann parents: 
45959diff
changeset | 1847 | |
| 46127 | 1848 | |
| 45959 
184d36538e51
`set` is now a proper type constructor; added operation for set monad
 haftmann parents: 
45909diff
changeset | 1849 | text {* Misc *}
 | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1850 | |
| 45152 | 1851 | hide_const (open) member not_member | 
| 32135 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1852 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1853 | lemmas equalityI = subset_antisym | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1854 | |
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1855 | ML {*
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1856 | val Ball_def = @{thm Ball_def}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1857 | val Bex_def = @{thm Bex_def}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1858 | val CollectD = @{thm CollectD}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1859 | val CollectE = @{thm CollectE}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1860 | val CollectI = @{thm CollectI}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1861 | val Collect_conj_eq = @{thm Collect_conj_eq}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1862 | val Collect_mem_eq = @{thm Collect_mem_eq}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1863 | val IntD1 = @{thm IntD1}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1864 | val IntD2 = @{thm IntD2}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1865 | val IntE = @{thm IntE}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1866 | val IntI = @{thm IntI}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1867 | val Int_Collect = @{thm Int_Collect}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1868 | val UNIV_I = @{thm UNIV_I}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1869 | val UNIV_witness = @{thm UNIV_witness}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1870 | val UnE = @{thm UnE}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1871 | val UnI1 = @{thm UnI1}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1872 | val UnI2 = @{thm UnI2}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1873 | val ballE = @{thm ballE}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1874 | val ballI = @{thm ballI}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1875 | val bexCI = @{thm bexCI}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1876 | val bexE = @{thm bexE}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1877 | val bexI = @{thm bexI}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1878 | val bex_triv = @{thm bex_triv}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1879 | val bspec = @{thm bspec}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1880 | val contra_subsetD = @{thm contra_subsetD}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1881 | val equalityCE = @{thm equalityCE}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1882 | val equalityD1 = @{thm equalityD1}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1883 | val equalityD2 = @{thm equalityD2}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1884 | val equalityE = @{thm equalityE}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1885 | val equalityI = @{thm equalityI}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1886 | val imageE = @{thm imageE}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1887 | val imageI = @{thm imageI}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1888 | val image_Un = @{thm image_Un}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1889 | val image_insert = @{thm image_insert}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1890 | val insert_commute = @{thm insert_commute}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1891 | val insert_iff = @{thm insert_iff}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1892 | val mem_Collect_eq = @{thm mem_Collect_eq}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1893 | val rangeE = @{thm rangeE}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1894 | val rangeI = @{thm rangeI}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1895 | val range_eqI = @{thm range_eqI}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1896 | val subsetCE = @{thm subsetCE}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1897 | val subsetD = @{thm subsetD}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1898 | val subsetI = @{thm subsetI}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1899 | val subset_refl = @{thm subset_refl}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1900 | val subset_trans = @{thm subset_trans}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1901 | val vimageD = @{thm vimageD}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1902 | val vimageE = @{thm vimageE}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1903 | val vimageI = @{thm vimageI}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1904 | val vimageI2 = @{thm vimageI2}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1905 | val vimage_Collect = @{thm vimage_Collect}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1906 | val vimage_Int = @{thm vimage_Int}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1907 | val vimage_Un = @{thm vimage_Un}
 | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1908 | *} | 
| 
f645b51e8e54
set intersection and union now named inter and union; closer connection between set and lattice operations; factored out complete lattice
 haftmann parents: 
32120diff
changeset | 1909 | |
| 32077 
3698947146b2
closer relation of sets and complete lattices; corresponding consts, defs and syntax at similar places in theory text
 haftmann parents: 
32064diff
changeset | 1910 | end | 
| 46853 | 1911 |