| author | wenzelm | 
| Mon, 15 Mar 2010 20:27:23 +0100 | |
| changeset 35799 | 7adb03f27b28 | 
| parent 35652 | 05ca920cd94b | 
| child 35900 | aa5dfb03eb1e | 
| permissions | -rw-r--r-- | 
| 33589 | 1 | (* Title: HOLCF/Representable.thy | 
| 2 | Author: Brian Huffman | |
| 3 | *) | |
| 4 | ||
| 33588 | 5 | header {* Representable Types *}
 | 
| 6 | ||
| 7 | theory Representable | |
| 35652 
05ca920cd94b
move take-proofs stuff into new theory Domain_Aux.thy
 huffman parents: 
35596diff
changeset | 8 | imports Algebraic Universal Ssum Sprod One Fixrec Domain_Aux | 
| 33794 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 9 | uses | 
| 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 10 |   ("Tools/repdef.ML")
 | 
| 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 11 |   ("Tools/Domain/domain_isomorphism.ML")
 | 
| 33588 | 12 | begin | 
| 13 | ||
| 14 | subsection {* Class of representable types *}
 | |
| 15 | ||
| 16 | text "Overloaded embedding and projection functions between | |
| 17 | a representable type and the universal domain." | |
| 18 | ||
| 19 | class rep = bifinite + | |
| 20 | fixes emb :: "'a::pcpo \<rightarrow> udom" | |
| 21 | fixes prj :: "udom \<rightarrow> 'a::pcpo" | |
| 22 | assumes ep_pair_emb_prj: "ep_pair emb prj" | |
| 23 | ||
| 24 | interpretation rep!: | |
| 25 | pcpo_ep_pair | |
| 26 | "emb :: 'a::rep \<rightarrow> udom" | |
| 27 | "prj :: udom \<rightarrow> 'a::rep" | |
| 28 | unfolding pcpo_ep_pair_def | |
| 29 | by (rule ep_pair_emb_prj) | |
| 30 | ||
| 31 | lemmas emb_inverse = rep.e_inverse | |
| 32 | lemmas emb_prj_below = rep.e_p_below | |
| 33 | lemmas emb_eq_iff = rep.e_eq_iff | |
| 34 | lemmas emb_strict = rep.e_strict | |
| 35 | lemmas prj_strict = rep.p_strict | |
| 36 | ||
| 37 | ||
| 38 | subsection {* Making @{term rep} the default class *}
 | |
| 39 | ||
| 40 | text {*
 | |
| 41 | From now on, free type variables are assumed to be in class | |
| 42 |   @{term rep}, unless specified otherwise.
 | |
| 43 | *} | |
| 44 | ||
| 45 | defaultsort rep | |
| 46 | ||
| 47 | subsection {* Representations of types *}
 | |
| 48 | ||
| 49 | text "A TypeRep is an algebraic deflation over the universe of values." | |
| 50 | ||
| 51 | types TypeRep = "udom alg_defl" | |
| 35431 | 52 | translations (type) "TypeRep" \<leftharpoondown> (type) "udom alg_defl" | 
| 33588 | 53 | |
| 54 | definition | |
| 55 | Rep_of :: "'a::rep itself \<Rightarrow> TypeRep" | |
| 56 | where | |
| 57 |   "Rep_of TYPE('a::rep) =
 | |
| 58 | (\<Squnion>i. alg_defl_principal (Abs_fin_defl | |
| 59 | (emb oo (approx i :: 'a \<rightarrow> 'a) oo prj)))" | |
| 60 | ||
| 61 | syntax "_REP" :: "type \<Rightarrow> TypeRep"  ("(1REP/(1'(_')))")
 | |
| 35431 | 62 | translations "REP('t)" \<rightleftharpoons> "CONST Rep_of TYPE('t)"
 | 
| 33588 | 63 | |
| 64 | lemma cast_REP: | |
| 65 |   "cast\<cdot>REP('a::rep) = (emb::'a \<rightarrow> udom) oo (prj::udom \<rightarrow> 'a)"
 | |
| 66 | proof - | |
| 67 | let ?a = "\<lambda>i. emb oo approx i oo (prj::udom \<rightarrow> 'a)" | |
| 68 | have a: "\<And>i. finite_deflation (?a i)" | |
| 69 | apply (rule rep.finite_deflation_e_d_p) | |
| 70 | apply (rule finite_deflation_approx) | |
| 71 | done | |
| 72 | show ?thesis | |
| 73 | unfolding Rep_of_def | |
| 74 | apply (subst contlub_cfun_arg) | |
| 75 | apply (rule chainI) | |
| 76 | apply (rule alg_defl.principal_mono) | |
| 77 | apply (rule Abs_fin_defl_mono [OF a a]) | |
| 78 | apply (rule chainE, simp) | |
| 79 | apply (subst cast_alg_defl_principal) | |
| 80 | apply (simp add: Abs_fin_defl_inverse a) | |
| 81 | apply (simp add: expand_cfun_eq lub_distribs) | |
| 82 | done | |
| 83 | qed | |
| 84 | ||
| 85 | lemma emb_prj: "emb\<cdot>((prj\<cdot>x)::'a::rep) = cast\<cdot>REP('a)\<cdot>x"
 | |
| 86 | by (simp add: cast_REP) | |
| 87 | ||
| 88 | lemma in_REP_iff: | |
| 89 |   "x ::: REP('a::rep) \<longleftrightarrow> emb\<cdot>((prj\<cdot>x)::'a) = x"
 | |
| 90 | by (simp add: in_deflation_def cast_REP) | |
| 91 | ||
| 92 | lemma prj_inverse: | |
| 93 |   "x ::: REP('a::rep) \<Longrightarrow> emb\<cdot>((prj\<cdot>x)::'a) = x"
 | |
| 94 | by (simp only: in_REP_iff) | |
| 95 | ||
| 96 | lemma emb_in_REP [simp]: | |
| 97 |   "emb\<cdot>(x::'a::rep) ::: REP('a)"
 | |
| 98 | by (simp add: in_REP_iff) | |
| 99 | ||
| 100 | subsection {* Coerce operator *}
 | |
| 101 | ||
| 102 | definition coerce :: "'a \<rightarrow> 'b" | |
| 103 | where "coerce = prj oo emb" | |
| 104 | ||
| 105 | lemma beta_coerce: "coerce\<cdot>x = prj\<cdot>(emb\<cdot>x)" | |
| 106 | by (simp add: coerce_def) | |
| 107 | ||
| 108 | lemma prj_emb: "prj\<cdot>(emb\<cdot>x) = coerce\<cdot>x" | |
| 109 | by (simp add: coerce_def) | |
| 110 | ||
| 111 | lemma coerce_strict [simp]: "coerce\<cdot>\<bottom> = \<bottom>" | |
| 112 | by (simp add: coerce_def) | |
| 113 | ||
| 114 | lemma coerce_eq_ID [simp]: "(coerce :: 'a \<rightarrow> 'a) = ID" | |
| 115 | by (rule ext_cfun, simp add: beta_coerce) | |
| 116 | ||
| 117 | lemma emb_coerce: | |
| 118 |   "REP('a) \<sqsubseteq> REP('b)
 | |
| 119 | \<Longrightarrow> emb\<cdot>((coerce::'a \<rightarrow> 'b)\<cdot>x) = emb\<cdot>x" | |
| 120 | apply (simp add: beta_coerce) | |
| 121 | apply (rule prj_inverse) | |
| 122 | apply (erule subdeflationD) | |
| 123 | apply (rule emb_in_REP) | |
| 124 | done | |
| 125 | ||
| 126 | lemma coerce_prj: | |
| 127 |   "REP('a) \<sqsubseteq> REP('b)
 | |
| 128 | \<Longrightarrow> (coerce::'b \<rightarrow> 'a)\<cdot>(prj\<cdot>x) = prj\<cdot>x" | |
| 129 | apply (simp add: coerce_def) | |
| 130 | apply (rule emb_eq_iff [THEN iffD1]) | |
| 131 | apply (simp only: emb_prj) | |
| 132 | apply (rule deflation_below_comp1) | |
| 133 | apply (rule deflation_cast) | |
| 134 | apply (rule deflation_cast) | |
| 135 | apply (erule monofun_cfun_arg) | |
| 136 | done | |
| 137 | ||
| 138 | lemma coerce_coerce [simp]: | |
| 139 |   "REP('a) \<sqsubseteq> REP('b)
 | |
| 140 | \<Longrightarrow> coerce\<cdot>((coerce::'a \<rightarrow> 'b)\<cdot>x) = coerce\<cdot>x" | |
| 141 | by (simp add: beta_coerce prj_inverse subdeflationD) | |
| 142 | ||
| 143 | lemma coerce_inverse: | |
| 144 |   "emb\<cdot>(x::'a) ::: REP('b) \<Longrightarrow> coerce\<cdot>(coerce\<cdot>x :: 'b) = x"
 | |
| 145 | by (simp only: beta_coerce prj_inverse emb_inverse) | |
| 146 | ||
| 147 | lemma coerce_type: | |
| 148 |   "REP('a) \<sqsubseteq> REP('b)
 | |
| 149 |    \<Longrightarrow> emb\<cdot>((coerce::'a \<rightarrow> 'b)\<cdot>x) ::: REP('a)"
 | |
| 150 | by (simp add: beta_coerce prj_inverse subdeflationD) | |
| 151 | ||
| 152 | lemma ep_pair_coerce: | |
| 153 |   "REP('a) \<sqsubseteq> REP('b)
 | |
| 154 | \<Longrightarrow> ep_pair (coerce::'a \<rightarrow> 'b) (coerce::'b \<rightarrow> 'a)" | |
| 155 | apply (rule ep_pair.intro) | |
| 156 | apply simp | |
| 157 | apply (simp only: beta_coerce) | |
| 158 | apply (rule below_trans) | |
| 159 | apply (rule monofun_cfun_arg) | |
| 160 | apply (rule emb_prj_below) | |
| 161 | apply simp | |
| 162 | done | |
| 163 | ||
| 33779 | 164 | text {* Isomorphism lemmas used internally by the domain package: *}
 | 
| 165 | ||
| 166 | lemma domain_abs_iso: | |
| 167 | fixes abs and rep | |
| 168 |   assumes REP: "REP('b) = REP('a)"
 | |
| 169 | assumes abs_def: "abs \<equiv> (coerce :: 'a \<rightarrow> 'b)" | |
| 170 | assumes rep_def: "rep \<equiv> (coerce :: 'b \<rightarrow> 'a)" | |
| 171 | shows "rep\<cdot>(abs\<cdot>x) = x" | |
| 172 | unfolding abs_def rep_def by (simp add: REP) | |
| 173 | ||
| 174 | lemma domain_rep_iso: | |
| 175 | fixes abs and rep | |
| 176 |   assumes REP: "REP('b) = REP('a)"
 | |
| 177 | assumes abs_def: "abs \<equiv> (coerce :: 'a \<rightarrow> 'b)" | |
| 178 | assumes rep_def: "rep \<equiv> (coerce :: 'b \<rightarrow> 'a)" | |
| 179 | shows "abs\<cdot>(rep\<cdot>x) = x" | |
| 180 | unfolding abs_def rep_def by (simp add: REP [symmetric]) | |
| 181 | ||
| 182 | ||
| 33588 | 183 | subsection {* Proving a subtype is representable *}
 | 
| 184 | ||
| 185 | text {*
 | |
| 186 |   Temporarily relax type constraints for @{term "approx"},
 | |
| 187 |   @{term emb}, and @{term prj}.
 | |
| 188 | *} | |
| 189 | ||
| 190 | setup {* Sign.add_const_constraint
 | |
| 191 |   (@{const_name "approx"}, SOME @{typ "nat \<Rightarrow> 'a::cpo \<rightarrow> 'a"}) *}
 | |
| 192 | ||
| 193 | setup {* Sign.add_const_constraint
 | |
| 194 |   (@{const_name emb}, SOME @{typ "'a::pcpo \<rightarrow> udom"}) *}
 | |
| 195 | ||
| 196 | setup {* Sign.add_const_constraint
 | |
| 197 |   (@{const_name prj}, SOME @{typ "udom \<rightarrow> 'a::pcpo"}) *}
 | |
| 198 | ||
| 33679 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 199 | definition | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 200 | repdef_approx :: | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 201 |     "('a::pcpo \<Rightarrow> udom) \<Rightarrow> (udom \<Rightarrow> 'a) \<Rightarrow> udom alg_defl \<Rightarrow> nat \<Rightarrow> 'a \<rightarrow> 'a"
 | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 202 | where | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 203 | "repdef_approx Rep Abs t = (\<lambda>i. \<Lambda> x. Abs (cast\<cdot>(approx i\<cdot>t)\<cdot>(Rep x)))" | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 204 | |
| 33588 | 205 | lemma typedef_rep_class: | 
| 206 | fixes Rep :: "'a::pcpo \<Rightarrow> udom" | |
| 207 | fixes Abs :: "udom \<Rightarrow> 'a::pcpo" | |
| 208 | fixes t :: TypeRep | |
| 209 |   assumes type: "type_definition Rep Abs {x. x ::: t}"
 | |
| 210 | assumes below: "op \<sqsubseteq> \<equiv> \<lambda>x y. Rep x \<sqsubseteq> Rep y" | |
| 33679 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 211 | assumes emb: "emb \<equiv> (\<Lambda> x. Rep x)" | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 212 | assumes prj: "prj \<equiv> (\<Lambda> x. Abs (cast\<cdot>t\<cdot>x))" | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 213 | assumes approx: "(approx :: nat \<Rightarrow> 'a \<rightarrow> 'a) \<equiv> repdef_approx Rep Abs t" | 
| 33588 | 214 |   shows "OFCLASS('a, rep_class)"
 | 
| 215 | proof | |
| 216 |   have adm: "adm (\<lambda>x. x \<in> {x. x ::: t})"
 | |
| 217 | by (simp add: adm_in_deflation) | |
| 218 | have emb_beta: "\<And>x. emb\<cdot>x = Rep x" | |
| 219 | unfolding emb | |
| 220 | apply (rule beta_cfun) | |
| 221 | apply (rule typedef_cont_Rep [OF type below adm]) | |
| 222 | done | |
| 223 | have prj_beta: "\<And>y. prj\<cdot>y = Abs (cast\<cdot>t\<cdot>y)" | |
| 224 | unfolding prj | |
| 225 | apply (rule beta_cfun) | |
| 226 | apply (rule typedef_cont_Abs [OF type below adm]) | |
| 227 | apply simp_all | |
| 228 | done | |
| 33679 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 229 | have cast_cast_approx: | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 230 | "\<And>i x. cast\<cdot>t\<cdot>(cast\<cdot>(approx i\<cdot>t)\<cdot>x) = cast\<cdot>(approx i\<cdot>t)\<cdot>x" | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 231 | apply (rule cast_fixed) | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 232 | apply (rule subdeflationD) | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 233 | apply (rule approx.below) | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 234 | apply (rule cast_in_deflation) | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 235 | done | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 236 | have approx': | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 237 | "approx = (\<lambda>i. \<Lambda>(x::'a). prj\<cdot>(cast\<cdot>(approx i\<cdot>t)\<cdot>(emb\<cdot>x)))" | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 238 | unfolding approx repdef_approx_def | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 239 | apply (subst cast_cast_approx [symmetric]) | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 240 | apply (simp add: prj_beta [symmetric] emb_beta [symmetric]) | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 241 | done | 
| 33588 | 242 | have emb_in_deflation: "\<And>x::'a. emb\<cdot>x ::: t" | 
| 243 | using type_definition.Rep [OF type] | |
| 244 | by (simp add: emb_beta) | |
| 245 | have prj_emb: "\<And>x::'a. prj\<cdot>(emb\<cdot>x) = x" | |
| 246 | unfolding prj_beta | |
| 247 | apply (simp add: cast_fixed [OF emb_in_deflation]) | |
| 248 | apply (simp add: emb_beta type_definition.Rep_inverse [OF type]) | |
| 249 | done | |
| 250 | have emb_prj: "\<And>y. emb\<cdot>(prj\<cdot>y :: 'a) = cast\<cdot>t\<cdot>y" | |
| 251 | unfolding prj_beta emb_beta | |
| 252 | by (simp add: type_definition.Abs_inverse [OF type]) | |
| 253 | show "ep_pair (emb :: 'a \<rightarrow> udom) prj" | |
| 254 | apply default | |
| 255 | apply (simp add: prj_emb) | |
| 256 | apply (simp add: emb_prj cast.below) | |
| 257 | done | |
| 258 | show "chain (approx :: nat \<Rightarrow> 'a \<rightarrow> 'a)" | |
| 33679 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 259 | unfolding approx' by simp | 
| 33588 | 260 | show "\<And>x::'a. (\<Squnion>i. approx i\<cdot>x) = x" | 
| 33679 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 261 | unfolding approx' | 
| 33588 | 262 | apply (simp add: lub_distribs) | 
| 263 | apply (subst cast_fixed [OF emb_in_deflation]) | |
| 264 | apply (rule prj_emb) | |
| 265 | done | |
| 266 | show "\<And>(i::nat) (x::'a). approx i\<cdot>(approx i\<cdot>x) = approx i\<cdot>x" | |
| 33679 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 267 | unfolding approx' | 
| 33588 | 268 | apply simp | 
| 269 | apply (simp add: emb_prj) | |
| 270 | apply (simp add: cast_cast_approx) | |
| 271 | done | |
| 272 |   show "\<And>i::nat. finite {x::'a. approx i\<cdot>x = x}"
 | |
| 273 |     apply (rule_tac B="(\<lambda>x. prj\<cdot>x) ` {x. cast\<cdot>(approx i\<cdot>t)\<cdot>x = x}"
 | |
| 274 | in finite_subset) | |
| 33679 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 275 | apply (clarsimp simp add: approx') | 
| 33588 | 276 | apply (drule_tac f="\<lambda>x. emb\<cdot>x" in arg_cong) | 
| 277 | apply (rule image_eqI) | |
| 278 | apply (rule prj_emb [symmetric]) | |
| 279 | apply (simp add: emb_prj) | |
| 280 | apply (simp add: cast_cast_approx) | |
| 281 | apply (rule finite_imageI) | |
| 282 | apply (simp add: cast_approx_fixed_iff) | |
| 283 | apply (simp add: Collect_conj_eq) | |
| 284 | apply (simp add: finite_fixes_approx) | |
| 285 | done | |
| 286 | qed | |
| 287 | ||
| 288 | text {* Restore original typing constraints *}
 | |
| 289 | ||
| 290 | setup {* Sign.add_const_constraint
 | |
| 291 |   (@{const_name "approx"}, SOME @{typ "nat \<Rightarrow> 'a::profinite \<rightarrow> 'a"}) *}
 | |
| 292 | ||
| 293 | setup {* Sign.add_const_constraint
 | |
| 294 |   (@{const_name emb}, SOME @{typ "'a::rep \<rightarrow> udom"}) *}
 | |
| 295 | ||
| 296 | setup {* Sign.add_const_constraint
 | |
| 297 |   (@{const_name prj}, SOME @{typ "udom \<rightarrow> 'a::rep"}) *}
 | |
| 298 | ||
| 299 | lemma typedef_REP: | |
| 300 | fixes Rep :: "'a::rep \<Rightarrow> udom" | |
| 301 | fixes Abs :: "udom \<Rightarrow> 'a::rep" | |
| 302 | fixes t :: TypeRep | |
| 303 |   assumes type: "type_definition Rep Abs {x. x ::: t}"
 | |
| 304 | assumes below: "op \<sqsubseteq> \<equiv> \<lambda>x y. Rep x \<sqsubseteq> Rep y" | |
| 33679 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 305 | assumes emb: "emb \<equiv> (\<Lambda> x. Rep x)" | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 306 | assumes prj: "prj \<equiv> (\<Lambda> x. Abs (cast\<cdot>t\<cdot>x))" | 
| 33588 | 307 |   shows "REP('a) = t"
 | 
| 308 | proof - | |
| 309 |   have adm: "adm (\<lambda>x. x \<in> {x. x ::: t})"
 | |
| 310 | by (simp add: adm_in_deflation) | |
| 311 | have emb_beta: "\<And>x. emb\<cdot>x = Rep x" | |
| 312 | unfolding emb | |
| 313 | apply (rule beta_cfun) | |
| 314 | apply (rule typedef_cont_Rep [OF type below adm]) | |
| 315 | done | |
| 316 | have prj_beta: "\<And>y. prj\<cdot>y = Abs (cast\<cdot>t\<cdot>y)" | |
| 317 | unfolding prj | |
| 318 | apply (rule beta_cfun) | |
| 319 | apply (rule typedef_cont_Abs [OF type below adm]) | |
| 320 | apply simp_all | |
| 321 | done | |
| 322 | have emb_in_deflation: "\<And>x::'a. emb\<cdot>x ::: t" | |
| 323 | using type_definition.Rep [OF type] | |
| 324 | by (simp add: emb_beta) | |
| 325 | have prj_emb: "\<And>x::'a. prj\<cdot>(emb\<cdot>x) = x" | |
| 326 | unfolding prj_beta | |
| 327 | apply (simp add: cast_fixed [OF emb_in_deflation]) | |
| 328 | apply (simp add: emb_beta type_definition.Rep_inverse [OF type]) | |
| 329 | done | |
| 330 | have emb_prj: "\<And>y. emb\<cdot>(prj\<cdot>y :: 'a) = cast\<cdot>t\<cdot>y" | |
| 331 | unfolding prj_beta emb_beta | |
| 332 | by (simp add: type_definition.Abs_inverse [OF type]) | |
| 333 |   show "REP('a) = t"
 | |
| 334 | apply (rule cast_eq_imp_eq, rule ext_cfun) | |
| 335 | apply (simp add: cast_REP emb_prj) | |
| 336 | done | |
| 337 | qed | |
| 338 | ||
| 33679 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 339 | lemma adm_mem_Collect_in_deflation: "adm (\<lambda>x. x \<in> {x. x ::: A})"
 | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 340 | unfolding mem_Collect_eq by (rule adm_in_deflation) | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 341 | |
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 342 | use "Tools/repdef.ML" | 
| 
331712879666
automate definition of representable domains from algebraic deflations
 huffman parents: 
33589diff
changeset | 343 | |
| 33588 | 344 | |
| 345 | subsection {* Instances of class @{text rep} *}
 | |
| 346 | ||
| 347 | subsubsection {* Universal Domain *}
 | |
| 348 | ||
| 349 | text "The Universal Domain itself is trivially representable." | |
| 350 | ||
| 351 | instantiation udom :: rep | |
| 352 | begin | |
| 353 | ||
| 354 | definition emb_udom_def [simp]: "emb = (ID :: udom \<rightarrow> udom)" | |
| 355 | definition prj_udom_def [simp]: "prj = (ID :: udom \<rightarrow> udom)" | |
| 356 | ||
| 357 | instance | |
| 358 | apply (intro_classes) | |
| 359 | apply (simp_all add: ep_pair.intro) | |
| 360 | done | |
| 361 | ||
| 362 | end | |
| 363 | ||
| 364 | subsubsection {* Lifted types *}
 | |
| 365 | ||
| 366 | instantiation lift :: (countable) rep | |
| 367 | begin | |
| 368 | ||
| 369 | definition emb_lift_def: | |
| 370 | "emb = udom_emb oo (FLIFT x. Def (to_nat x))" | |
| 371 | ||
| 372 | definition prj_lift_def: | |
| 373 | "prj = (FLIFT n. if (\<exists>x::'a::countable. n = to_nat x) | |
| 374 | then Def (THE x::'a. n = to_nat x) else \<bottom>) oo udom_prj" | |
| 375 | ||
| 376 | instance | |
| 377 | apply (intro_classes, unfold emb_lift_def prj_lift_def) | |
| 378 | apply (rule ep_pair_comp [OF _ ep_pair_udom]) | |
| 379 | apply (rule ep_pair.intro) | |
| 380 | apply (case_tac x, simp, simp) | |
| 381 | apply (case_tac y, simp, clarsimp) | |
| 382 | done | |
| 383 | ||
| 384 | end | |
| 385 | ||
| 386 | subsubsection {* Representable type constructors *}
 | |
| 387 | ||
| 388 | text "Functions between representable types are representable." | |
| 389 | ||
| 35525 | 390 | instantiation cfun :: (rep, rep) rep | 
| 33588 | 391 | begin | 
| 392 | ||
| 393 | definition emb_cfun_def: "emb = udom_emb oo cfun_map\<cdot>prj\<cdot>emb" | |
| 394 | definition prj_cfun_def: "prj = cfun_map\<cdot>emb\<cdot>prj oo udom_prj" | |
| 395 | ||
| 396 | instance | |
| 397 | apply (intro_classes, unfold emb_cfun_def prj_cfun_def) | |
| 398 | apply (intro ep_pair_comp ep_pair_cfun_map ep_pair_emb_prj ep_pair_udom) | |
| 399 | done | |
| 400 | ||
| 401 | end | |
| 402 | ||
| 403 | text "Strict products of representable types are representable." | |
| 404 | ||
| 35525 | 405 | instantiation sprod :: (rep, rep) rep | 
| 33588 | 406 | begin | 
| 407 | ||
| 408 | definition emb_sprod_def: "emb = udom_emb oo sprod_map\<cdot>emb\<cdot>emb" | |
| 409 | definition prj_sprod_def: "prj = sprod_map\<cdot>prj\<cdot>prj oo udom_prj" | |
| 410 | ||
| 411 | instance | |
| 412 | apply (intro_classes, unfold emb_sprod_def prj_sprod_def) | |
| 413 | apply (intro ep_pair_comp ep_pair_sprod_map ep_pair_emb_prj ep_pair_udom) | |
| 414 | done | |
| 415 | ||
| 416 | end | |
| 417 | ||
| 418 | text "Strict sums of representable types are representable." | |
| 419 | ||
| 35525 | 420 | instantiation ssum :: (rep, rep) rep | 
| 33588 | 421 | begin | 
| 422 | ||
| 423 | definition emb_ssum_def: "emb = udom_emb oo ssum_map\<cdot>emb\<cdot>emb" | |
| 424 | definition prj_ssum_def: "prj = ssum_map\<cdot>prj\<cdot>prj oo udom_prj" | |
| 425 | ||
| 426 | instance | |
| 427 | apply (intro_classes, unfold emb_ssum_def prj_ssum_def) | |
| 428 | apply (intro ep_pair_comp ep_pair_ssum_map ep_pair_emb_prj ep_pair_udom) | |
| 429 | done | |
| 430 | ||
| 431 | end | |
| 432 | ||
| 433 | text "Up of a representable type is representable." | |
| 434 | ||
| 435 | instantiation "u" :: (rep) rep | |
| 436 | begin | |
| 437 | ||
| 438 | definition emb_u_def: "emb = udom_emb oo u_map\<cdot>emb" | |
| 439 | definition prj_u_def: "prj = u_map\<cdot>prj oo udom_prj" | |
| 440 | ||
| 441 | instance | |
| 442 | apply (intro_classes, unfold emb_u_def prj_u_def) | |
| 443 | apply (intro ep_pair_comp ep_pair_u_map ep_pair_emb_prj ep_pair_udom) | |
| 444 | done | |
| 445 | ||
| 446 | end | |
| 447 | ||
| 448 | text "Cartesian products of representable types are representable." | |
| 449 | ||
| 450 | instantiation "*" :: (rep, rep) rep | |
| 451 | begin | |
| 452 | ||
| 453 | definition emb_cprod_def: "emb = udom_emb oo cprod_map\<cdot>emb\<cdot>emb" | |
| 454 | definition prj_cprod_def: "prj = cprod_map\<cdot>prj\<cdot>prj oo udom_prj" | |
| 455 | ||
| 456 | instance | |
| 457 | apply (intro_classes, unfold emb_cprod_def prj_cprod_def) | |
| 458 | apply (intro ep_pair_comp ep_pair_cprod_map ep_pair_emb_prj ep_pair_udom) | |
| 459 | done | |
| 460 | ||
| 461 | end | |
| 462 | ||
| 463 | subsection {* Type combinators *}
 | |
| 464 | ||
| 465 | definition | |
| 466 | TypeRep_fun1 :: | |
| 467 |     "((udom \<rightarrow> udom) \<rightarrow> ('a \<rightarrow> 'a))
 | |
| 468 | \<Rightarrow> (TypeRep \<rightarrow> TypeRep)" | |
| 469 | where | |
| 470 | "TypeRep_fun1 f = | |
| 471 | alg_defl.basis_fun (\<lambda>a. | |
| 472 | alg_defl_principal ( | |
| 473 | Abs_fin_defl (udom_emb oo f\<cdot>(Rep_fin_defl a) oo udom_prj)))" | |
| 474 | ||
| 475 | definition | |
| 476 | TypeRep_fun2 :: | |
| 477 |     "((udom \<rightarrow> udom) \<rightarrow> (udom \<rightarrow> udom) \<rightarrow> ('a \<rightarrow> 'a))
 | |
| 478 | \<Rightarrow> (TypeRep \<rightarrow> TypeRep \<rightarrow> TypeRep)" | |
| 479 | where | |
| 480 | "TypeRep_fun2 f = | |
| 481 | alg_defl.basis_fun (\<lambda>a. | |
| 482 | alg_defl.basis_fun (\<lambda>b. | |
| 483 | alg_defl_principal ( | |
| 484 | Abs_fin_defl (udom_emb oo | |
| 485 | f\<cdot>(Rep_fin_defl a)\<cdot>(Rep_fin_defl b) oo udom_prj))))" | |
| 486 | ||
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 487 | definition "cfun_defl = TypeRep_fun2 cfun_map" | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 488 | definition "ssum_defl = TypeRep_fun2 ssum_map" | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 489 | definition "sprod_defl = TypeRep_fun2 sprod_map" | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 490 | definition "cprod_defl = TypeRep_fun2 cprod_map" | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 491 | definition "u_defl = TypeRep_fun1 u_map" | 
| 33588 | 492 | |
| 493 | lemma Rep_fin_defl_mono: "a \<sqsubseteq> b \<Longrightarrow> Rep_fin_defl a \<sqsubseteq> Rep_fin_defl b" | |
| 494 | unfolding below_fin_defl_def . | |
| 495 | ||
| 496 | lemma cast_TypeRep_fun1: | |
| 497 | assumes f: "\<And>a. finite_deflation a \<Longrightarrow> finite_deflation (f\<cdot>a)" | |
| 498 | shows "cast\<cdot>(TypeRep_fun1 f\<cdot>A) = udom_emb oo f\<cdot>(cast\<cdot>A) oo udom_prj" | |
| 499 | proof - | |
| 500 | have 1: "\<And>a. finite_deflation (udom_emb oo f\<cdot>(Rep_fin_defl a) oo udom_prj)" | |
| 501 | apply (rule ep_pair.finite_deflation_e_d_p [OF ep_pair_udom]) | |
| 502 | apply (rule f, rule finite_deflation_Rep_fin_defl) | |
| 503 | done | |
| 504 | show ?thesis | |
| 505 | by (induct A rule: alg_defl.principal_induct, simp) | |
| 506 | (simp only: TypeRep_fun1_def | |
| 507 | alg_defl.basis_fun_principal | |
| 508 | alg_defl.basis_fun_mono | |
| 509 | alg_defl.principal_mono | |
| 510 | Abs_fin_defl_mono [OF 1 1] | |
| 511 | monofun_cfun below_refl | |
| 512 | Rep_fin_defl_mono | |
| 513 | cast_alg_defl_principal | |
| 514 | Abs_fin_defl_inverse [unfolded mem_Collect_eq, OF 1]) | |
| 515 | qed | |
| 516 | ||
| 517 | lemma cast_TypeRep_fun2: | |
| 518 | assumes f: "\<And>a b. finite_deflation a \<Longrightarrow> finite_deflation b \<Longrightarrow> | |
| 519 | finite_deflation (f\<cdot>a\<cdot>b)" | |
| 520 | shows "cast\<cdot>(TypeRep_fun2 f\<cdot>A\<cdot>B) = udom_emb oo f\<cdot>(cast\<cdot>A)\<cdot>(cast\<cdot>B) oo udom_prj" | |
| 521 | proof - | |
| 522 | have 1: "\<And>a b. finite_deflation | |
| 523 | (udom_emb oo f\<cdot>(Rep_fin_defl a)\<cdot>(Rep_fin_defl b) oo udom_prj)" | |
| 524 | apply (rule ep_pair.finite_deflation_e_d_p [OF ep_pair_udom]) | |
| 525 | apply (rule f, (rule finite_deflation_Rep_fin_defl)+) | |
| 526 | done | |
| 527 | show ?thesis | |
| 528 | by (induct A B rule: alg_defl.principal_induct2, simp, simp) | |
| 529 | (simp only: TypeRep_fun2_def | |
| 530 | alg_defl.basis_fun_principal | |
| 531 | alg_defl.basis_fun_mono | |
| 532 | alg_defl.principal_mono | |
| 533 | Abs_fin_defl_mono [OF 1 1] | |
| 534 | monofun_cfun below_refl | |
| 535 | Rep_fin_defl_mono | |
| 536 | cast_alg_defl_principal | |
| 537 | Abs_fin_defl_inverse [unfolded mem_Collect_eq, OF 1]) | |
| 538 | qed | |
| 539 | ||
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 540 | lemma cast_cfun_defl: | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 541 | "cast\<cdot>(cfun_defl\<cdot>A\<cdot>B) = udom_emb oo cfun_map\<cdot>(cast\<cdot>A)\<cdot>(cast\<cdot>B) oo udom_prj" | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 542 | unfolding cfun_defl_def | 
| 33588 | 543 | apply (rule cast_TypeRep_fun2) | 
| 544 | apply (erule (1) finite_deflation_cfun_map) | |
| 545 | done | |
| 546 | ||
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 547 | lemma cast_ssum_defl: | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 548 | "cast\<cdot>(ssum_defl\<cdot>A\<cdot>B) = udom_emb oo ssum_map\<cdot>(cast\<cdot>A)\<cdot>(cast\<cdot>B) oo udom_prj" | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 549 | unfolding ssum_defl_def | 
| 33588 | 550 | apply (rule cast_TypeRep_fun2) | 
| 551 | apply (erule (1) finite_deflation_ssum_map) | |
| 552 | done | |
| 553 | ||
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 554 | lemma cast_sprod_defl: | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 555 | "cast\<cdot>(sprod_defl\<cdot>A\<cdot>B) = udom_emb oo sprod_map\<cdot>(cast\<cdot>A)\<cdot>(cast\<cdot>B) oo udom_prj" | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 556 | unfolding sprod_defl_def | 
| 33588 | 557 | apply (rule cast_TypeRep_fun2) | 
| 558 | apply (erule (1) finite_deflation_sprod_map) | |
| 559 | done | |
| 560 | ||
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 561 | lemma cast_cprod_defl: | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 562 | "cast\<cdot>(cprod_defl\<cdot>A\<cdot>B) = udom_emb oo cprod_map\<cdot>(cast\<cdot>A)\<cdot>(cast\<cdot>B) oo udom_prj" | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 563 | unfolding cprod_defl_def | 
| 33588 | 564 | apply (rule cast_TypeRep_fun2) | 
| 565 | apply (erule (1) finite_deflation_cprod_map) | |
| 566 | done | |
| 567 | ||
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 568 | lemma cast_u_defl: | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 569 | "cast\<cdot>(u_defl\<cdot>A) = udom_emb oo u_map\<cdot>(cast\<cdot>A) oo udom_prj" | 
| 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 570 | unfolding u_defl_def | 
| 33588 | 571 | apply (rule cast_TypeRep_fun1) | 
| 572 | apply (erule finite_deflation_u_map) | |
| 573 | done | |
| 574 | ||
| 575 | text {* REP of type constructor = type combinator *}
 | |
| 576 | ||
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 577 | lemma REP_cfun: "REP('a \<rightarrow> 'b) = cfun_defl\<cdot>REP('a)\<cdot>REP('b)"
 | 
| 33588 | 578 | apply (rule cast_eq_imp_eq, rule ext_cfun) | 
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 579 | apply (simp add: cast_REP cast_cfun_defl) | 
| 33588 | 580 | apply (simp add: cfun_map_def) | 
| 581 | apply (simp only: prj_cfun_def emb_cfun_def) | |
| 582 | apply (simp add: expand_cfun_eq ep_pair.e_eq_iff [OF ep_pair_udom]) | |
| 583 | done | |
| 584 | ||
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 585 | lemma REP_ssum: "REP('a \<oplus> 'b) = ssum_defl\<cdot>REP('a)\<cdot>REP('b)"
 | 
| 33588 | 586 | apply (rule cast_eq_imp_eq, rule ext_cfun) | 
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 587 | apply (simp add: cast_REP cast_ssum_defl) | 
| 33588 | 588 | apply (simp add: prj_ssum_def) | 
| 589 | apply (simp add: emb_ssum_def) | |
| 590 | apply (simp add: ssum_map_map cfcomp1) | |
| 591 | done | |
| 592 | ||
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 593 | lemma REP_sprod: "REP('a \<otimes> 'b) = sprod_defl\<cdot>REP('a)\<cdot>REP('b)"
 | 
| 33588 | 594 | apply (rule cast_eq_imp_eq, rule ext_cfun) | 
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 595 | apply (simp add: cast_REP cast_sprod_defl) | 
| 33588 | 596 | apply (simp add: prj_sprod_def) | 
| 597 | apply (simp add: emb_sprod_def) | |
| 598 | apply (simp add: sprod_map_map cfcomp1) | |
| 599 | done | |
| 600 | ||
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 601 | lemma REP_cprod: "REP('a \<times> 'b) = cprod_defl\<cdot>REP('a)\<cdot>REP('b)"
 | 
| 33588 | 602 | apply (rule cast_eq_imp_eq, rule ext_cfun) | 
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 603 | apply (simp add: cast_REP cast_cprod_defl) | 
| 33588 | 604 | apply (simp add: prj_cprod_def) | 
| 605 | apply (simp add: emb_cprod_def) | |
| 606 | apply (simp add: cprod_map_map cfcomp1) | |
| 607 | done | |
| 608 | ||
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 609 | lemma REP_up: "REP('a u) = u_defl\<cdot>REP('a)"
 | 
| 33588 | 610 | apply (rule cast_eq_imp_eq, rule ext_cfun) | 
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 611 | apply (simp add: cast_REP cast_u_defl) | 
| 33588 | 612 | apply (simp add: prj_u_def) | 
| 613 | apply (simp add: emb_u_def) | |
| 614 | apply (simp add: u_map_map cfcomp1) | |
| 615 | done | |
| 616 | ||
| 617 | lemmas REP_simps = | |
| 618 | REP_cfun | |
| 619 | REP_ssum | |
| 620 | REP_sprod | |
| 621 | REP_cprod | |
| 622 | REP_up | |
| 623 | ||
| 624 | subsection {* Isomorphic deflations *}
 | |
| 625 | ||
| 626 | definition | |
| 627 |   isodefl :: "('a::rep \<rightarrow> 'a) \<Rightarrow> udom alg_defl \<Rightarrow> bool"
 | |
| 628 | where | |
| 629 | "isodefl d t \<longleftrightarrow> cast\<cdot>t = emb oo d oo prj" | |
| 630 | ||
| 631 | lemma isodeflI: "(\<And>x. cast\<cdot>t\<cdot>x = emb\<cdot>(d\<cdot>(prj\<cdot>x))) \<Longrightarrow> isodefl d t" | |
| 632 | unfolding isodefl_def by (simp add: ext_cfun) | |
| 633 | ||
| 634 | lemma cast_isodefl: "isodefl d t \<Longrightarrow> cast\<cdot>t = (\<Lambda> x. emb\<cdot>(d\<cdot>(prj\<cdot>x)))" | |
| 635 | unfolding isodefl_def by (simp add: ext_cfun) | |
| 636 | ||
| 637 | lemma isodefl_strict: "isodefl d t \<Longrightarrow> d\<cdot>\<bottom> = \<bottom>" | |
| 638 | unfolding isodefl_def | |
| 639 | by (drule cfun_fun_cong [where x="\<bottom>"], simp) | |
| 640 | ||
| 641 | lemma isodefl_imp_deflation: | |
| 642 | fixes d :: "'a::rep \<rightarrow> 'a" | |
| 643 | assumes "isodefl d t" shows "deflation d" | |
| 644 | proof | |
| 645 | note prems [unfolded isodefl_def, simp] | |
| 646 | fix x :: 'a | |
| 647 | show "d\<cdot>(d\<cdot>x) = d\<cdot>x" | |
| 648 | using cast.idem [of t "emb\<cdot>x"] by simp | |
| 649 | show "d\<cdot>x \<sqsubseteq> x" | |
| 650 | using cast.below [of t "emb\<cdot>x"] by simp | |
| 651 | qed | |
| 652 | ||
| 653 | lemma isodefl_ID_REP: "isodefl (ID :: 'a \<rightarrow> 'a) REP('a)"
 | |
| 654 | unfolding isodefl_def by (simp add: cast_REP) | |
| 655 | ||
| 656 | lemma isodefl_REP_imp_ID: "isodefl (d :: 'a \<rightarrow> 'a) REP('a) \<Longrightarrow> d = ID"
 | |
| 657 | unfolding isodefl_def | |
| 658 | apply (simp add: cast_REP) | |
| 659 | apply (simp add: expand_cfun_eq) | |
| 660 | apply (rule allI) | |
| 661 | apply (drule_tac x="emb\<cdot>x" in spec) | |
| 662 | apply simp | |
| 663 | done | |
| 664 | ||
| 665 | lemma isodefl_bottom: "isodefl \<bottom> \<bottom>" | |
| 666 | unfolding isodefl_def by (simp add: expand_cfun_eq) | |
| 667 | ||
| 668 | lemma adm_isodefl: | |
| 669 | "cont f \<Longrightarrow> cont g \<Longrightarrow> adm (\<lambda>x. isodefl (f x) (g x))" | |
| 670 | unfolding isodefl_def by simp | |
| 671 | ||
| 672 | lemma isodefl_lub: | |
| 673 | assumes "chain d" and "chain t" | |
| 674 | assumes "\<And>i. isodefl (d i) (t i)" | |
| 675 | shows "isodefl (\<Squnion>i. d i) (\<Squnion>i. t i)" | |
| 676 | using prems unfolding isodefl_def | |
| 677 | by (simp add: contlub_cfun_arg contlub_cfun_fun) | |
| 678 | ||
| 679 | lemma isodefl_fix: | |
| 680 | assumes "\<And>d t. isodefl d t \<Longrightarrow> isodefl (f\<cdot>d) (g\<cdot>t)" | |
| 681 | shows "isodefl (fix\<cdot>f) (fix\<cdot>g)" | |
| 682 | unfolding fix_def2 | |
| 683 | apply (rule isodefl_lub, simp, simp) | |
| 684 | apply (induct_tac i) | |
| 685 | apply (simp add: isodefl_bottom) | |
| 686 | apply (simp add: prems) | |
| 687 | done | |
| 688 | ||
| 689 | lemma isodefl_coerce: | |
| 690 | fixes d :: "'a \<rightarrow> 'a" | |
| 691 |   assumes REP: "REP('b) = REP('a)"
 | |
| 692 | shows "isodefl d t \<Longrightarrow> isodefl (coerce oo d oo coerce :: 'b \<rightarrow> 'b) t" | |
| 693 | unfolding isodefl_def | |
| 694 | apply (simp add: expand_cfun_eq) | |
| 695 | apply (simp add: emb_coerce coerce_prj REP) | |
| 696 | done | |
| 697 | ||
| 33779 | 698 | lemma isodefl_abs_rep: | 
| 699 | fixes abs and rep and d | |
| 700 |   assumes REP: "REP('b) = REP('a)"
 | |
| 701 | assumes abs_def: "abs \<equiv> (coerce :: 'a \<rightarrow> 'b)" | |
| 702 | assumes rep_def: "rep \<equiv> (coerce :: 'b \<rightarrow> 'a)" | |
| 703 | shows "isodefl d t \<Longrightarrow> isodefl (abs oo d oo rep) t" | |
| 704 | unfolding abs_def rep_def using REP by (rule isodefl_coerce) | |
| 705 | ||
| 33588 | 706 | lemma isodefl_cfun: | 
| 707 | "isodefl d1 t1 \<Longrightarrow> isodefl d2 t2 \<Longrightarrow> | |
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 708 | isodefl (cfun_map\<cdot>d1\<cdot>d2) (cfun_defl\<cdot>t1\<cdot>t2)" | 
| 33588 | 709 | apply (rule isodeflI) | 
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 710 | apply (simp add: cast_cfun_defl cast_isodefl) | 
| 33588 | 711 | apply (simp add: emb_cfun_def prj_cfun_def) | 
| 712 | apply (simp add: cfun_map_map cfcomp1) | |
| 713 | done | |
| 714 | ||
| 715 | lemma isodefl_ssum: | |
| 716 | "isodefl d1 t1 \<Longrightarrow> isodefl d2 t2 \<Longrightarrow> | |
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 717 | isodefl (ssum_map\<cdot>d1\<cdot>d2) (ssum_defl\<cdot>t1\<cdot>t2)" | 
| 33588 | 718 | apply (rule isodeflI) | 
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 719 | apply (simp add: cast_ssum_defl cast_isodefl) | 
| 33588 | 720 | apply (simp add: emb_ssum_def prj_ssum_def) | 
| 721 | apply (simp add: ssum_map_map isodefl_strict) | |
| 722 | done | |
| 723 | ||
| 724 | lemma isodefl_sprod: | |
| 725 | "isodefl d1 t1 \<Longrightarrow> isodefl d2 t2 \<Longrightarrow> | |
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 726 | isodefl (sprod_map\<cdot>d1\<cdot>d2) (sprod_defl\<cdot>t1\<cdot>t2)" | 
| 33588 | 727 | apply (rule isodeflI) | 
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 728 | apply (simp add: cast_sprod_defl cast_isodefl) | 
| 33588 | 729 | apply (simp add: emb_sprod_def prj_sprod_def) | 
| 730 | apply (simp add: sprod_map_map isodefl_strict) | |
| 731 | done | |
| 732 | ||
| 33786 | 733 | lemma isodefl_cprod: | 
| 734 | "isodefl d1 t1 \<Longrightarrow> isodefl d2 t2 \<Longrightarrow> | |
| 735 | isodefl (cprod_map\<cdot>d1\<cdot>d2) (cprod_defl\<cdot>t1\<cdot>t2)" | |
| 736 | apply (rule isodeflI) | |
| 737 | apply (simp add: cast_cprod_defl cast_isodefl) | |
| 738 | apply (simp add: emb_cprod_def prj_cprod_def) | |
| 739 | apply (simp add: cprod_map_map cfcomp1) | |
| 740 | done | |
| 741 | ||
| 33588 | 742 | lemma isodefl_u: | 
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 743 | "isodefl d t \<Longrightarrow> isodefl (u_map\<cdot>d) (u_defl\<cdot>t)" | 
| 33588 | 744 | apply (rule isodeflI) | 
| 33784 
7e434813752f
change naming convention for deflation combinators
 huffman parents: 
33779diff
changeset | 745 | apply (simp add: cast_u_defl cast_isodefl) | 
| 33588 | 746 | apply (simp add: emb_u_def prj_u_def) | 
| 747 | apply (simp add: u_map_map) | |
| 748 | done | |
| 749 | ||
| 33794 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 750 | subsection {* Constructing Domain Isomorphisms *}
 | 
| 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 751 | |
| 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 752 | use "Tools/Domain/domain_isomorphism.ML" | 
| 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 753 | |
| 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 754 | setup {*
 | 
| 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 755 | fold Domain_Isomorphism.add_type_constructor | 
| 35525 | 756 |     [(@{type_name cfun}, @{term cfun_defl}, @{const_name cfun_map}, @{thm REP_cfun},
 | 
| 35479 
dffffe36344a
store deflation thms for map functions in theory data
 huffman parents: 
35475diff
changeset | 757 |         @{thm isodefl_cfun}, @{thm cfun_map_ID}, @{thm deflation_cfun_map}),
 | 
| 33794 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 758 | |
| 35525 | 759 |      (@{type_name ssum}, @{term ssum_defl}, @{const_name ssum_map}, @{thm REP_ssum},
 | 
| 35479 
dffffe36344a
store deflation thms for map functions in theory data
 huffman parents: 
35475diff
changeset | 760 |         @{thm isodefl_ssum}, @{thm ssum_map_ID}, @{thm deflation_ssum_map}),
 | 
| 33794 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 761 | |
| 35525 | 762 |      (@{type_name sprod}, @{term sprod_defl}, @{const_name sprod_map}, @{thm REP_sprod},
 | 
| 35479 
dffffe36344a
store deflation thms for map functions in theory data
 huffman parents: 
35475diff
changeset | 763 |         @{thm isodefl_sprod}, @{thm sprod_map_ID}, @{thm deflation_sprod_map}),
 | 
| 33794 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 764 | |
| 35479 
dffffe36344a
store deflation thms for map functions in theory data
 huffman parents: 
35475diff
changeset | 765 |      (@{type_name "*"}, @{term cprod_defl}, @{const_name cprod_map}, @{thm REP_cprod},
 | 
| 
dffffe36344a
store deflation thms for map functions in theory data
 huffman parents: 
35475diff
changeset | 766 |         @{thm isodefl_cprod}, @{thm cprod_map_ID}, @{thm deflation_cprod_map}),
 | 
| 33794 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 767 | |
| 35479 
dffffe36344a
store deflation thms for map functions in theory data
 huffman parents: 
35475diff
changeset | 768 |      (@{type_name "u"}, @{term u_defl}, @{const_name u_map}, @{thm REP_up},
 | 
| 
dffffe36344a
store deflation thms for map functions in theory data
 huffman parents: 
35475diff
changeset | 769 |         @{thm isodefl_u}, @{thm u_map_ID}, @{thm deflation_u_map})]
 | 
| 33794 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 770 | *} | 
| 
364bc92ba081
set up domain_isomorphism package in Representable.thy
 huffman parents: 
33786diff
changeset | 771 | |
| 33588 | 772 | end |