author | haftmann |
Thu, 19 Jun 2025 17:15:40 +0200 | |
changeset 82734 | 89347c0cc6a3 |
parent 81583 | b6df83045178 |
permissions | -rw-r--r-- |
42151 | 1 |
(* Title: HOL/HOLCF/Lift.thy |
72835 | 2 |
Author: Olaf Müller |
2640 | 3 |
*) |
4 |
||
62175 | 5 |
section \<open>Lifting types of class type to flat pcpo's\<close> |
12026 | 6 |
|
15577 | 7 |
theory Lift |
81575 | 8 |
imports Up |
15577 | 9 |
begin |
12026 | 10 |
|
81583
b6df83045178
clarified default_sort: "cpo" for bootstrap, "domain" for main HOLCF;
wenzelm
parents:
81577
diff
changeset
|
11 |
pcpodef 'a::type lift = "UNIV :: 'a discr u set" |
29063
7619f0561cd7
pcpodef package: state two goals, instead of encoded conjunction;
wenzelm
parents:
27311
diff
changeset
|
12 |
by simp_all |
12026 | 13 |
|
16748 | 14 |
lemmas inst_lift_pcpo = Abs_lift_strict [symmetric] |
12026 | 15 |
|
25131
2c8caac48ade
modernized specifications ('definition', 'abbreviation', 'notation');
wenzelm
parents:
19764
diff
changeset
|
16 |
definition |
81583
b6df83045178
clarified default_sort: "cpo" for bootstrap, "domain" for main HOLCF;
wenzelm
parents:
81577
diff
changeset
|
17 |
Def :: "'a::type \<Rightarrow> 'a lift" where |
25131
2c8caac48ade
modernized specifications ('definition', 'abbreviation', 'notation');
wenzelm
parents:
19764
diff
changeset
|
18 |
"Def x = Abs_lift (up\<cdot>(Discr x))" |
12026 | 19 |
|
81577 | 20 |
|
62175 | 21 |
subsection \<open>Lift as a datatype\<close> |
12026 | 22 |
|
16748 | 23 |
lemma lift_induct: "\<lbrakk>P \<bottom>; \<And>x. P (Def x)\<rbrakk> \<Longrightarrow> P y" |
24 |
apply (induct y) |
|
16755
fd02f9d06e43
renamed upE1 to upE; added simp rule cont2cont_flift1
huffman
parents:
16749
diff
changeset
|
25 |
apply (rule_tac p=y in upE) |
16748 | 26 |
apply (simp add: Abs_lift_strict) |
27 |
apply (case_tac x) |
|
28 |
apply (simp add: Def_def) |
|
29 |
done |
|
12026 | 30 |
|
81583
b6df83045178
clarified default_sort: "cpo" for bootstrap, "domain" for main HOLCF;
wenzelm
parents:
81577
diff
changeset
|
31 |
old_rep_datatype "\<bottom>::'a::type lift" Def |
40082 | 32 |
by (erule lift_induct) (simp_all add: Def_def Abs_lift_inject inst_lift_pcpo) |
12026 | 33 |
|
69597 | 34 |
text \<open>\<^term>\<open>bottom\<close> and \<^term>\<open>Def\<close>\<close> |
12026 | 35 |
|
16748 | 36 |
lemma not_Undef_is_Def: "(x \<noteq> \<bottom>) = (\<exists>y. x = Def y)" |
12026 | 37 |
by (cases x) simp_all |
38 |
||
16630
83bf468b1dc7
added theorem lift_definedE; moved cont_if to Cont.thy
huffman
parents:
16555
diff
changeset
|
39 |
lemma lift_definedE: "\<lbrakk>x \<noteq> \<bottom>; \<And>a. x = Def a \<Longrightarrow> R\<rbrakk> \<Longrightarrow> R" |
83bf468b1dc7
added theorem lift_definedE; moved cont_if to Cont.thy
huffman
parents:
16555
diff
changeset
|
40 |
by (cases x) simp_all |
83bf468b1dc7
added theorem lift_definedE; moved cont_if to Cont.thy
huffman
parents:
16555
diff
changeset
|
41 |
|
62175 | 42 |
text \<open> |
69597 | 43 |
For \<^term>\<open>x ~= \<bottom>\<close> in assumptions \<open>defined\<close> replaces \<open>x\<close> by \<open>Def a\<close> in conclusion.\<close> |
12026 | 44 |
|
62175 | 45 |
method_setup defined = \<open> |
30607
c3d1590debd8
eliminated global SIMPSET, CLASET etc. -- refer to explicit context;
wenzelm
parents:
29138
diff
changeset
|
46 |
Scan.succeed (fn ctxt => SIMPLE_METHOD' |
60754 | 47 |
(eresolve_tac ctxt @{thms lift_definedE} THEN' asm_simp_tac ctxt)) |
62175 | 48 |
\<close> |
12026 | 49 |
|
16748 | 50 |
lemma DefE: "Def x = \<bottom> \<Longrightarrow> R" |
51 |
by simp |
|
12026 | 52 |
|
16748 | 53 |
lemma DefE2: "\<lbrakk>x = Def s; x = \<bottom>\<rbrakk> \<Longrightarrow> R" |
12026 | 54 |
by simp |
55 |
||
31076
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
huffman
parents:
30607
diff
changeset
|
56 |
lemma Def_below_Def: "Def x \<sqsubseteq> Def y \<longleftrightarrow> x = y" |
40082 | 57 |
by (simp add: below_lift_def Def_def Abs_lift_inverse) |
12026 | 58 |
|
31076
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
huffman
parents:
30607
diff
changeset
|
59 |
lemma Def_below_iff [simp]: "Def x \<sqsubseteq> y \<longleftrightarrow> Def x = y" |
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
huffman
parents:
30607
diff
changeset
|
60 |
by (induct y, simp, simp add: Def_below_Def) |
12026 | 61 |
|
62 |
||
62175 | 63 |
subsection \<open>Lift is flat\<close> |
12026 | 64 |
|
12338
de0f4a63baa5
renamed class "term" to "type" (actually "HOL.type");
wenzelm
parents:
12026
diff
changeset
|
65 |
instance lift :: (type) flat |
27292 | 66 |
proof |
67 |
fix x y :: "'a lift" |
|
68 |
assume "x \<sqsubseteq> y" thus "x = \<bottom> \<or> x = y" |
|
69 |
by (induct x) auto |
|
70 |
qed |
|
12026 | 71 |
|
81577 | 72 |
|
69597 | 73 |
subsection \<open>Continuity of \<^const>\<open>case_lift\<close>\<close> |
40088
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
74 |
|
55417
01fbfb60c33e
adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems
blanchet
parents:
51717
diff
changeset
|
75 |
lemma case_lift_eq: "case_lift \<bottom> f x = fup\<cdot>(\<Lambda> y. f (undiscr y))\<cdot>(Rep_lift x)" |
55642
63beb38e9258
adapted to renaming of datatype 'cases' and 'recs' to 'case' and 'rec'
blanchet
parents:
55417
diff
changeset
|
76 |
apply (induct x, unfold lift.case) |
40088
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
77 |
apply (simp add: Rep_lift_strict) |
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
78 |
apply (simp add: Def_def Abs_lift_inverse) |
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
79 |
done |
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
80 |
|
55417
01fbfb60c33e
adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems
blanchet
parents:
51717
diff
changeset
|
81 |
lemma cont2cont_case_lift [simp]: |
01fbfb60c33e
adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems
blanchet
parents:
51717
diff
changeset
|
82 |
"\<lbrakk>\<And>y. cont (\<lambda>x. f x y); cont g\<rbrakk> \<Longrightarrow> cont (\<lambda>x. case_lift \<bottom> (f x) (g x))" |
01fbfb60c33e
adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems
blanchet
parents:
51717
diff
changeset
|
83 |
unfolding case_lift_eq by (simp add: cont_Rep_lift) |
40088
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
84 |
|
81577 | 85 |
|
62175 | 86 |
subsection \<open>Further operations\<close> |
16695
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
87 |
|
25131
2c8caac48ade
modernized specifications ('definition', 'abbreviation', 'notation');
wenzelm
parents:
19764
diff
changeset
|
88 |
definition |
81583
b6df83045178
clarified default_sort: "cpo" for bootstrap, "domain" for main HOLCF;
wenzelm
parents:
81577
diff
changeset
|
89 |
flift1 :: "('a::type \<Rightarrow> 'b::pcpo) \<Rightarrow> ('a lift \<rightarrow> 'b)" (binder \<open>FLIFT \<close> 10) where |
55417
01fbfb60c33e
adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems
blanchet
parents:
51717
diff
changeset
|
90 |
"flift1 = (\<lambda>f. (\<Lambda> x. case_lift \<bottom> f x))" |
16695
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
91 |
|
40323
4cce7c708402
add 'LAM (Def x). t' as alternative syntax for 'FLIFT x. t'
huffman
parents:
40321
diff
changeset
|
92 |
translations |
4cce7c708402
add 'LAM (Def x). t' as alternative syntax for 'FLIFT x. t'
huffman
parents:
40321
diff
changeset
|
93 |
"\<Lambda>(XCONST Def x). t" => "CONST flift1 (\<lambda>x. t)" |
4cce7c708402
add 'LAM (Def x). t' as alternative syntax for 'FLIFT x. t'
huffman
parents:
40321
diff
changeset
|
94 |
"\<Lambda>(CONST Def x). FLIFT y. t" <= "FLIFT x y. t" |
4cce7c708402
add 'LAM (Def x). t' as alternative syntax for 'FLIFT x. t'
huffman
parents:
40321
diff
changeset
|
95 |
"\<Lambda>(CONST Def x). t" <= "FLIFT x. t" |
4cce7c708402
add 'LAM (Def x). t' as alternative syntax for 'FLIFT x. t'
huffman
parents:
40321
diff
changeset
|
96 |
|
25131
2c8caac48ade
modernized specifications ('definition', 'abbreviation', 'notation');
wenzelm
parents:
19764
diff
changeset
|
97 |
definition |
81583
b6df83045178
clarified default_sort: "cpo" for bootstrap, "domain" for main HOLCF;
wenzelm
parents:
81577
diff
changeset
|
98 |
flift2 :: "('a::type \<Rightarrow> 'b::type) \<Rightarrow> ('a lift \<rightarrow> 'b lift)" where |
25131
2c8caac48ade
modernized specifications ('definition', 'abbreviation', 'notation');
wenzelm
parents:
19764
diff
changeset
|
99 |
"flift2 f = (FLIFT x. Def (f x))" |
16695
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
100 |
|
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
101 |
lemma flift1_Def [simp]: "flift1 f\<cdot>(Def x) = (f x)" |
40088
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
102 |
by (simp add: flift1_def) |
16695
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
103 |
|
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
104 |
lemma flift2_Def [simp]: "flift2 f\<cdot>(Def x) = Def (f x)" |
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
105 |
by (simp add: flift2_def) |
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
106 |
|
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
107 |
lemma flift1_strict [simp]: "flift1 f\<cdot>\<bottom> = \<bottom>" |
40088
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
108 |
by (simp add: flift1_def) |
16695
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
109 |
|
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
110 |
lemma flift2_strict [simp]: "flift2 f\<cdot>\<bottom> = \<bottom>" |
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
111 |
by (simp add: flift2_def) |
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
112 |
|
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
113 |
lemma flift2_defined [simp]: "x \<noteq> \<bottom> \<Longrightarrow> (flift2 f)\<cdot>x \<noteq> \<bottom>" |
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
114 |
by (erule lift_definedE, simp) |
dc8c868e910b
simplified definitions of flift1, flift2, liftpair;
huffman
parents:
16630
diff
changeset
|
115 |
|
40321
d065b195ec89
rename lemmas *_defined_iff and *_strict_iff to *_bottom_iff
huffman
parents:
40089
diff
changeset
|
116 |
lemma flift2_bottom_iff [simp]: "(flift2 f\<cdot>x = \<bottom>) = (x = \<bottom>)" |
19520 | 117 |
by (cases x, simp_all) |
118 |
||
40088
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
119 |
lemma FLIFT_mono: |
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
120 |
"(\<And>x. f x \<sqsubseteq> g x) \<Longrightarrow> (FLIFT x. f x) \<sqsubseteq> (FLIFT x. g x)" |
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
121 |
by (rule cfun_belowI, case_tac x, simp_all) |
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
122 |
|
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
123 |
lemma cont2cont_flift1 [simp, cont2cont]: |
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
124 |
"\<lbrakk>\<And>y. cont (\<lambda>x. f x y)\<rbrakk> \<Longrightarrow> cont (\<lambda>x. FLIFT y. f x y)" |
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
125 |
by (simp add: flift1_def cont2cont_LAM) |
49b9d301fadb
simplify proofs about flift; remove unneeded lemmas
huffman
parents:
40086
diff
changeset
|
126 |
|
2640 | 127 |
end |