author | wenzelm |
Fri, 08 Dec 2023 13:09:39 +0100 | |
changeset 79198 | 2586c8b422ed |
parent 69712 | dc85b5b3a532 |
permissions | -rw-r--r-- |
43158 | 1 |
(* Author: Tobias Nipkow *) |
2 |
||
58889 | 3 |
section "Live Variable Analysis" |
43158 | 4 |
|
5 |
theory Live imports Vars Big_Step |
|
6 |
begin |
|
7 |
||
8 |
subsection "Liveness Analysis" |
|
9 |
||
45212 | 10 |
fun L :: "com \<Rightarrow> vname set \<Rightarrow> vname set" where |
51425 | 11 |
"L SKIP X = X" | |
51448 | 12 |
"L (x ::= a) X = vars a \<union> (X - {x})" | |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52046
diff
changeset
|
13 |
"L (c\<^sub>1;; c\<^sub>2) X = L c\<^sub>1 (L c\<^sub>2 X)" | |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52046
diff
changeset
|
14 |
"L (IF b THEN c\<^sub>1 ELSE c\<^sub>2) X = vars b \<union> L c\<^sub>1 X \<union> L c\<^sub>2 X" | |
51425 | 15 |
"L (WHILE b DO c) X = vars b \<union> X \<union> L c X" |
43158 | 16 |
|
52046
bc01725d7918
replaced `;' by `;;' to disambiguate syntax; unexpected slight increase in build time
nipkow
parents:
51975
diff
changeset
|
17 |
value "show (L (''y'' ::= V ''z'';; ''x'' ::= Plus (V ''y'') (V ''z'')) {''x''})" |
43158 | 18 |
|
19 |
value "show (L (WHILE Less (V ''x'') (V ''x'') DO ''y'' ::= V ''z'') {''x''})" |
|
20 |
||
45212 | 21 |
fun "kill" :: "com \<Rightarrow> vname set" where |
43158 | 22 |
"kill SKIP = {}" | |
23 |
"kill (x ::= a) = {x}" | |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52046
diff
changeset
|
24 |
"kill (c\<^sub>1;; c\<^sub>2) = kill c\<^sub>1 \<union> kill c\<^sub>2" | |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52046
diff
changeset
|
25 |
"kill (IF b THEN c\<^sub>1 ELSE c\<^sub>2) = kill c\<^sub>1 \<inter> kill c\<^sub>2" | |
43158 | 26 |
"kill (WHILE b DO c) = {}" |
27 |
||
45212 | 28 |
fun gen :: "com \<Rightarrow> vname set" where |
43158 | 29 |
"gen SKIP = {}" | |
30 |
"gen (x ::= a) = vars a" | |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52046
diff
changeset
|
31 |
"gen (c\<^sub>1;; c\<^sub>2) = gen c\<^sub>1 \<union> (gen c\<^sub>2 - kill c\<^sub>1)" | |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52046
diff
changeset
|
32 |
"gen (IF b THEN c\<^sub>1 ELSE c\<^sub>2) = vars b \<union> gen c\<^sub>1 \<union> gen c\<^sub>2" | |
43158 | 33 |
"gen (WHILE b DO c) = vars b \<union> gen c" |
34 |
||
51433 | 35 |
lemma L_gen_kill: "L c X = gen c \<union> (X - kill c)" |
43158 | 36 |
by(induct c arbitrary:X) auto |
37 |
||
45771 | 38 |
lemma L_While_pfp: "L c (L (WHILE b DO c) X) \<subseteq> L (WHILE b DO c) X" |
43158 | 39 |
by(auto simp add:L_gen_kill) |
40 |
||
45771 | 41 |
lemma L_While_lpfp: |
45784 | 42 |
"vars b \<union> X \<union> L c P \<subseteq> P \<Longrightarrow> L (WHILE b DO c) X \<subseteq> P" |
45771 | 43 |
by(simp add: L_gen_kill) |
44 |
||
51468
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
45 |
lemma L_While_vars: "vars b \<subseteq> L (WHILE b DO c) X" |
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
46 |
by auto |
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
47 |
|
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
48 |
lemma L_While_X: "X \<subseteq> L (WHILE b DO c) X" |
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
49 |
by auto |
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
50 |
|
67406 | 51 |
text\<open>Disable L WHILE equation and reason only with L WHILE constraints\<close> |
51468
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
52 |
declare L.simps(5)[simp del] |
43158 | 53 |
|
51975 | 54 |
subsection "Correctness" |
43158 | 55 |
|
51975 | 56 |
theorem L_correct: |
43158 | 57 |
"(c,s) \<Rightarrow> s' \<Longrightarrow> s = t on L c X \<Longrightarrow> |
58 |
\<exists> t'. (c,t) \<Rightarrow> t' & s' = t' on X" |
|
45015 | 59 |
proof (induction arbitrary: X t rule: big_step_induct) |
43158 | 60 |
case Skip then show ?case by auto |
61 |
next |
|
62 |
case Assign then show ?case |
|
63 |
by (auto simp: ball_Un) |
|
64 |
next |
|
47818 | 65 |
case (Seq c1 s1 s2 c2 s3 X t1) |
66 |
from Seq.IH(1) Seq.prems obtain t2 where |
|
43158 | 67 |
t12: "(c1, t1) \<Rightarrow> t2" and s2t2: "s2 = t2 on L c2 X" |
68 |
by simp blast |
|
47818 | 69 |
from Seq.IH(2)[OF s2t2] obtain t3 where |
43158 | 70 |
t23: "(c2, t2) \<Rightarrow> t3" and s3t3: "s3 = t3 on X" |
71 |
by auto |
|
72 |
show ?case using t12 t23 s3t3 by auto |
|
73 |
next |
|
74 |
case (IfTrue b s c1 s' c2) |
|
75 |
hence "s = t on vars b" "s = t on L c1 X" by auto |
|
76 |
from bval_eq_if_eq_on_vars[OF this(1)] IfTrue(1) have "bval b t" by simp |
|
67406 | 77 |
from IfTrue.IH[OF \<open>s = t on L c1 X\<close>] obtain t' where |
43158 | 78 |
"(c1, t) \<Rightarrow> t'" "s' = t' on X" by auto |
67406 | 79 |
thus ?case using \<open>bval b t\<close> by auto |
43158 | 80 |
next |
81 |
case (IfFalse b s c2 s' c1) |
|
82 |
hence "s = t on vars b" "s = t on L c2 X" by auto |
|
83 |
from bval_eq_if_eq_on_vars[OF this(1)] IfFalse(1) have "~bval b t" by simp |
|
67406 | 84 |
from IfFalse.IH[OF \<open>s = t on L c2 X\<close>] obtain t' where |
43158 | 85 |
"(c2, t) \<Rightarrow> t'" "s' = t' on X" by auto |
67406 | 86 |
thus ?case using \<open>~bval b t\<close> by auto |
43158 | 87 |
next |
88 |
case (WhileFalse b s c) |
|
51468
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
89 |
hence "~ bval b t" |
69712 | 90 |
by (metis L_While_vars bval_eq_if_eq_on_vars subsetD) |
91 |
thus ?case by(metis WhileFalse.prems L_While_X big_step.WhileFalse subsetD) |
|
43158 | 92 |
next |
93 |
case (WhileTrue b s1 c s2 s3 X t1) |
|
94 |
let ?w = "WHILE b DO c" |
|
67406 | 95 |
from \<open>bval b s1\<close> WhileTrue.prems have "bval b t1" |
69712 | 96 |
by (metis L_While_vars bval_eq_if_eq_on_vars subsetD) |
51468
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
97 |
have "s1 = t1 on L c (L ?w X)" using L_While_pfp WhileTrue.prems |
43158 | 98 |
by (blast) |
45015 | 99 |
from WhileTrue.IH(1)[OF this] obtain t2 where |
43158 | 100 |
"(c, t1) \<Rightarrow> t2" "s2 = t2 on L ?w X" by auto |
45015 | 101 |
from WhileTrue.IH(2)[OF this(2)] obtain t3 where "(?w,t2) \<Rightarrow> t3" "s3 = t3 on X" |
43158 | 102 |
by auto |
67406 | 103 |
with \<open>bval b t1\<close> \<open>(c, t1) \<Rightarrow> t2\<close> show ?case by auto |
43158 | 104 |
qed |
105 |
||
106 |
||
107 |
subsection "Program Optimization" |
|
108 |
||
67406 | 109 |
text\<open>Burying assignments to dead variables:\<close> |
45212 | 110 |
fun bury :: "com \<Rightarrow> vname set \<Rightarrow> com" where |
43158 | 111 |
"bury SKIP X = SKIP" | |
50009 | 112 |
"bury (x ::= a) X = (if x \<in> X then x ::= a else SKIP)" | |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52046
diff
changeset
|
113 |
"bury (c\<^sub>1;; c\<^sub>2) X = (bury c\<^sub>1 (L c\<^sub>2 X);; bury c\<^sub>2 X)" | |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52046
diff
changeset
|
114 |
"bury (IF b THEN c\<^sub>1 ELSE c\<^sub>2) X = IF b THEN bury c\<^sub>1 X ELSE bury c\<^sub>2 X" | |
51468
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
115 |
"bury (WHILE b DO c) X = WHILE b DO bury c (L (WHILE b DO c) X)" |
43158 | 116 |
|
67406 | 117 |
text\<open>We could prove the analogous lemma to @{thm[source]L_correct}, and the |
43158 | 118 |
proof would be very similar. However, we phrase it as a semantics |
67406 | 119 |
preservation property:\<close> |
43158 | 120 |
|
51975 | 121 |
theorem bury_correct: |
43158 | 122 |
"(c,s) \<Rightarrow> s' \<Longrightarrow> s = t on L c X \<Longrightarrow> |
123 |
\<exists> t'. (bury c X,t) \<Rightarrow> t' & s' = t' on X" |
|
45015 | 124 |
proof (induction arbitrary: X t rule: big_step_induct) |
43158 | 125 |
case Skip then show ?case by auto |
126 |
next |
|
127 |
case Assign then show ?case |
|
128 |
by (auto simp: ball_Un) |
|
129 |
next |
|
47818 | 130 |
case (Seq c1 s1 s2 c2 s3 X t1) |
131 |
from Seq.IH(1) Seq.prems obtain t2 where |
|
43158 | 132 |
t12: "(bury c1 (L c2 X), t1) \<Rightarrow> t2" and s2t2: "s2 = t2 on L c2 X" |
133 |
by simp blast |
|
47818 | 134 |
from Seq.IH(2)[OF s2t2] obtain t3 where |
43158 | 135 |
t23: "(bury c2 X, t2) \<Rightarrow> t3" and s3t3: "s3 = t3 on X" |
136 |
by auto |
|
137 |
show ?case using t12 t23 s3t3 by auto |
|
138 |
next |
|
139 |
case (IfTrue b s c1 s' c2) |
|
140 |
hence "s = t on vars b" "s = t on L c1 X" by auto |
|
141 |
from bval_eq_if_eq_on_vars[OF this(1)] IfTrue(1) have "bval b t" by simp |
|
67406 | 142 |
from IfTrue.IH[OF \<open>s = t on L c1 X\<close>] obtain t' where |
43158 | 143 |
"(bury c1 X, t) \<Rightarrow> t'" "s' =t' on X" by auto |
67406 | 144 |
thus ?case using \<open>bval b t\<close> by auto |
43158 | 145 |
next |
146 |
case (IfFalse b s c2 s' c1) |
|
147 |
hence "s = t on vars b" "s = t on L c2 X" by auto |
|
148 |
from bval_eq_if_eq_on_vars[OF this(1)] IfFalse(1) have "~bval b t" by simp |
|
67406 | 149 |
from IfFalse.IH[OF \<open>s = t on L c2 X\<close>] obtain t' where |
43158 | 150 |
"(bury c2 X, t) \<Rightarrow> t'" "s' = t' on X" by auto |
67406 | 151 |
thus ?case using \<open>~bval b t\<close> by auto |
43158 | 152 |
next |
153 |
case (WhileFalse b s c) |
|
69712 | 154 |
hence "~ bval b t" by (metis L_While_vars bval_eq_if_eq_on_vars subsetD) |
51468
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
155 |
thus ?case |
69712 | 156 |
by simp (metis L_While_X WhileFalse.prems big_step.WhileFalse subsetD) |
43158 | 157 |
next |
158 |
case (WhileTrue b s1 c s2 s3 X t1) |
|
159 |
let ?w = "WHILE b DO c" |
|
67406 | 160 |
from \<open>bval b s1\<close> WhileTrue.prems have "bval b t1" |
69712 | 161 |
by (metis L_While_vars bval_eq_if_eq_on_vars subsetD) |
43158 | 162 |
have "s1 = t1 on L c (L ?w X)" |
45771 | 163 |
using L_While_pfp WhileTrue.prems by blast |
45015 | 164 |
from WhileTrue.IH(1)[OF this] obtain t2 where |
43158 | 165 |
"(bury c (L ?w X), t1) \<Rightarrow> t2" "s2 = t2 on L ?w X" by auto |
45015 | 166 |
from WhileTrue.IH(2)[OF this(2)] obtain t3 |
43158 | 167 |
where "(bury ?w X,t2) \<Rightarrow> t3" "s3 = t3 on X" |
168 |
by auto |
|
67406 | 169 |
with \<open>bval b t1\<close> \<open>(bury c (L ?w X), t1) \<Rightarrow> t2\<close> show ?case by auto |
43158 | 170 |
qed |
171 |
||
51975 | 172 |
corollary final_bury_correct: "(c,s) \<Rightarrow> s' \<Longrightarrow> (bury c UNIV,s) \<Rightarrow> s'" |
173 |
using bury_correct[of c s s' UNIV] |
|
43158 | 174 |
by (auto simp: fun_eq_iff[symmetric]) |
175 |
||
67406 | 176 |
text\<open>Now the opposite direction.\<close> |
43158 | 177 |
|
178 |
lemma SKIP_bury[simp]: |
|
67613 | 179 |
"SKIP = bury c X \<longleftrightarrow> c = SKIP | (\<exists>x a. c = x::=a & x \<notin> X)" |
43158 | 180 |
by (cases c) auto |
181 |
||
67613 | 182 |
lemma Assign_bury[simp]: "x::=a = bury c X \<longleftrightarrow> c = x::=a \<and> x \<in> X" |
43158 | 183 |
by (cases c) auto |
184 |
||
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52046
diff
changeset
|
185 |
lemma Seq_bury[simp]: "bc\<^sub>1;;bc\<^sub>2 = bury c X \<longleftrightarrow> |
67613 | 186 |
(\<exists>c\<^sub>1 c\<^sub>2. c = c\<^sub>1;;c\<^sub>2 & bc\<^sub>2 = bury c\<^sub>2 X & bc\<^sub>1 = bury c\<^sub>1 (L c\<^sub>2 X))" |
43158 | 187 |
by (cases c) auto |
188 |
||
189 |
lemma If_bury[simp]: "IF b THEN bc1 ELSE bc2 = bury c X \<longleftrightarrow> |
|
67613 | 190 |
(\<exists>c1 c2. c = IF b THEN c1 ELSE c2 & |
43158 | 191 |
bc1 = bury c1 X & bc2 = bury c2 X)" |
192 |
by (cases c) auto |
|
193 |
||
194 |
lemma While_bury[simp]: "WHILE b DO bc' = bury c X \<longleftrightarrow> |
|
67613 | 195 |
(\<exists>c'. c = WHILE b DO c' & bc' = bury c' (L (WHILE b DO c') X))" |
43158 | 196 |
by (cases c) auto |
197 |
||
51975 | 198 |
theorem bury_correct2: |
43158 | 199 |
"(bury c X,s) \<Rightarrow> s' \<Longrightarrow> s = t on L c X \<Longrightarrow> |
200 |
\<exists> t'. (c,t) \<Rightarrow> t' & s' = t' on X" |
|
45015 | 201 |
proof (induction "bury c X" s s' arbitrary: c X t rule: big_step_induct) |
43158 | 202 |
case Skip then show ?case by auto |
203 |
next |
|
204 |
case Assign then show ?case |
|
205 |
by (auto simp: ball_Un) |
|
206 |
next |
|
47818 | 207 |
case (Seq bc1 s1 s2 bc2 s3 c X t1) |
52046
bc01725d7918
replaced `;' by `;;' to disambiguate syntax; unexpected slight increase in build time
nipkow
parents:
51975
diff
changeset
|
208 |
then obtain c1 c2 where c: "c = c1;;c2" |
43158 | 209 |
and bc2: "bc2 = bury c2 X" and bc1: "bc1 = bury c1 (L c2 X)" by auto |
47818 | 210 |
note IH = Seq.hyps(2,4) |
211 |
from IH(1)[OF bc1, of t1] Seq.prems c obtain t2 where |
|
43158 | 212 |
t12: "(c1, t1) \<Rightarrow> t2" and s2t2: "s2 = t2 on L c2 X" by auto |
45015 | 213 |
from IH(2)[OF bc2 s2t2] obtain t3 where |
43158 | 214 |
t23: "(c2, t2) \<Rightarrow> t3" and s3t3: "s3 = t3 on X" |
215 |
by auto |
|
216 |
show ?case using c t12 t23 s3t3 by auto |
|
217 |
next |
|
218 |
case (IfTrue b s bc1 s' bc2) |
|
219 |
then obtain c1 c2 where c: "c = IF b THEN c1 ELSE c2" |
|
220 |
and bc1: "bc1 = bury c1 X" and bc2: "bc2 = bury c2 X" by auto |
|
221 |
have "s = t on vars b" "s = t on L c1 X" using IfTrue.prems c by auto |
|
222 |
from bval_eq_if_eq_on_vars[OF this(1)] IfTrue(1) have "bval b t" by simp |
|
45015 | 223 |
note IH = IfTrue.hyps(3) |
67406 | 224 |
from IH[OF bc1 \<open>s = t on L c1 X\<close>] obtain t' where |
43158 | 225 |
"(c1, t) \<Rightarrow> t'" "s' =t' on X" by auto |
67406 | 226 |
thus ?case using c \<open>bval b t\<close> by auto |
43158 | 227 |
next |
228 |
case (IfFalse b s bc2 s' bc1) |
|
229 |
then obtain c1 c2 where c: "c = IF b THEN c1 ELSE c2" |
|
230 |
and bc1: "bc1 = bury c1 X" and bc2: "bc2 = bury c2 X" by auto |
|
231 |
have "s = t on vars b" "s = t on L c2 X" using IfFalse.prems c by auto |
|
232 |
from bval_eq_if_eq_on_vars[OF this(1)] IfFalse(1) have "~bval b t" by simp |
|
45015 | 233 |
note IH = IfFalse.hyps(3) |
67406 | 234 |
from IH[OF bc2 \<open>s = t on L c2 X\<close>] obtain t' where |
43158 | 235 |
"(c2, t) \<Rightarrow> t'" "s' =t' on X" by auto |
67406 | 236 |
thus ?case using c \<open>~bval b t\<close> by auto |
43158 | 237 |
next |
238 |
case (WhileFalse b s c) |
|
51468
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
239 |
hence "~ bval b t" |
69712 | 240 |
by auto (metis L_While_vars bval_eq_if_eq_on_vars rev_subsetD) |
51468
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
241 |
thus ?case using WhileFalse |
69712 | 242 |
by auto (metis L_While_X big_step.WhileFalse subsetD) |
43158 | 243 |
next |
51468
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
244 |
case (WhileTrue b s1 bc' s2 s3 w X t1) |
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
245 |
then obtain c' where w: "w = WHILE b DO c'" |
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
246 |
and bc': "bc' = bury c' (L (WHILE b DO c') X)" by auto |
67406 | 247 |
from \<open>bval b s1\<close> WhileTrue.prems w have "bval b t1" |
69712 | 248 |
by auto (metis L_While_vars bval_eq_if_eq_on_vars subsetD) |
45015 | 249 |
note IH = WhileTrue.hyps(3,5) |
51468
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
250 |
have "s1 = t1 on L c' (L w X)" |
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
251 |
using L_While_pfp WhileTrue.prems w by blast |
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
252 |
with IH(1)[OF bc', of t1] w obtain t2 where |
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
253 |
"(c', t1) \<Rightarrow> t2" "s2 = t2 on L w X" by auto |
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
254 |
from IH(2)[OF WhileTrue.hyps(6), of t2] w this(2) obtain t3 |
0e8012983c4e
proofs depend only on constraints, not on def of L WHILE
nipkow
parents:
51448
diff
changeset
|
255 |
where "(w,t2) \<Rightarrow> t3" "s3 = t3 on X" |
43158 | 256 |
by auto |
67406 | 257 |
with \<open>bval b t1\<close> \<open>(c', t1) \<Rightarrow> t2\<close> w show ?case by auto |
43158 | 258 |
qed |
259 |
||
51975 | 260 |
corollary final_bury_correct2: "(bury c UNIV,s) \<Rightarrow> s' \<Longrightarrow> (c,s) \<Rightarrow> s'" |
261 |
using bury_correct2[of c UNIV] |
|
43158 | 262 |
by (auto simp: fun_eq_iff[symmetric]) |
263 |
||
51433 | 264 |
corollary bury_sim: "bury c UNIV \<sim> c" |
51975 | 265 |
by(metis final_bury_correct final_bury_correct2) |
43158 | 266 |
|
267 |
end |