author | wenzelm |
Tue, 13 Aug 2013 22:37:58 +0200 | |
changeset 53024 | e0968e1f6fe9 |
parent 52866 | 438f578ef1d9 |
child 56073 | 29e308b56d23 |
permissions | -rw-r--r-- |
13673 | 1 |
(* Title: HOL/MicroJava/Comp/CorrComp.thy |
2 |
Author: Martin Strecker |
|
3 |
*) |
|
4 |
||
5 |
(* Compiler correctness statement and proof *) |
|
6 |
||
15860 | 7 |
theory CorrComp |
15866 | 8 |
imports "../J/JTypeSafe" "LemmasComp" |
15860 | 9 |
begin |
13673 | 10 |
|
14045 | 11 |
declare wf_prog_ws_prog [simp add] |
13673 | 12 |
|
13 |
(* If no exception is present after evaluation/execution, |
|
14 |
none can have been present before *) |
|
15 |
lemma eval_evals_exec_xcpt: |
|
22271 | 16 |
"(G \<turnstile> xs -ex\<succ>val-> xs' \<longrightarrow> gx xs' = None \<longrightarrow> gx xs = None) \<and> |
17 |
(G \<turnstile> xs -exs[\<succ>]vals-> xs' \<longrightarrow> gx xs' = None \<longrightarrow> gx xs = None) \<and> |
|
18 |
(G \<turnstile> xs -st-> xs' \<longrightarrow> gx xs' = None \<longrightarrow> gx xs = None)" |
|
52866 | 19 |
by (induct rule: eval_evals_exec.induct) auto |
13673 | 20 |
|
21 |
||
22 |
(* instance of eval_evals_exec_xcpt for eval *) |
|
22271 | 23 |
lemma eval_xcpt: "G \<turnstile> xs -ex\<succ>val-> xs' \<Longrightarrow> gx xs' = None \<Longrightarrow> gx xs = None" |
13673 | 24 |
(is "?H1 \<Longrightarrow> ?H2 \<Longrightarrow> ?T") |
25 |
proof- |
|
26 |
assume h1: ?H1 |
|
27 |
assume h2: ?H2 |
|
28 |
from h1 h2 eval_evals_exec_xcpt show "?T" by simp |
|
29 |
qed |
|
30 |
||
31 |
(* instance of eval_evals_exec_xcpt for evals *) |
|
22271 | 32 |
lemma evals_xcpt: "G \<turnstile> xs -exs[\<succ>]vals-> xs' \<Longrightarrow> gx xs' = None \<Longrightarrow> gx xs = None" |
13673 | 33 |
(is "?H1 \<Longrightarrow> ?H2 \<Longrightarrow> ?T") |
34 |
proof- |
|
35 |
assume h1: ?H1 |
|
36 |
assume h2: ?H2 |
|
37 |
from h1 h2 eval_evals_exec_xcpt show "?T" by simp |
|
38 |
qed |
|
39 |
||
40 |
(* instance of eval_evals_exec_xcpt for exec *) |
|
22271 | 41 |
lemma exec_xcpt: "G \<turnstile> xs -st-> xs' \<Longrightarrow> gx xs' = None \<Longrightarrow> gx xs = None" |
13673 | 42 |
(is "?H1 \<Longrightarrow> ?H2 \<Longrightarrow> ?T") |
43 |
proof- |
|
44 |
assume h1: ?H1 |
|
45 |
assume h2: ?H2 |
|
46 |
from h1 h2 eval_evals_exec_xcpt show "?T" by simp |
|
47 |
qed |
|
48 |
||
49 |
(**********************************************************************) |
|
50 |
||
51 |
theorem exec_all_trans: "\<lbrakk>(exec_all G s0 s1); (exec_all G s1 s2)\<rbrakk> \<Longrightarrow> (exec_all G s0 s2)" |
|
52 |
apply (auto simp: exec_all_def elim: Transitive_Closure.rtrancl_trans) |
|
53 |
done |
|
54 |
||
55 |
theorem exec_all_refl: "exec_all G s s" |
|
15097
b807858b97bd
Modifications for trancl_tac (new solver in simplifier).
ballarin
parents:
15076
diff
changeset
|
56 |
by (simp only: exec_all_def) |
13673 | 57 |
|
58 |
||
59 |
theorem exec_instr_in_exec_all: |
|
60 |
"\<lbrakk> exec_instr i G hp stk lvars C S pc frs = (None, hp', frs'); |
|
61 |
gis (gmb G C S) ! pc = i\<rbrakk> \<Longrightarrow> |
|
53024 | 62 |
G \<turnstile> (None, hp, (stk, lvars, C, S, pc) # frs) \<midarrow>jvm\<rightarrow> (None, hp', frs')" |
13673 | 63 |
apply (simp only: exec_all_def) |
64 |
apply (rule rtrancl_refl [THEN rtrancl_into_rtrancl]) |
|
65 |
apply (simp add: gis_def gmb_def) |
|
66 |
apply (case_tac frs', simp+) |
|
67 |
done |
|
68 |
||
69 |
theorem exec_all_one_step: " |
|
70 |
\<lbrakk> gis (gmb G C S) = pre @ (i # post); pc0 = length pre; |
|
71 |
(exec_instr i G hp0 stk0 lvars0 C S pc0 frs) = |
|
72 |
(None, hp1, (stk1,lvars1,C,S, Suc pc0)#frs) \<rbrakk> |
|
73 |
\<Longrightarrow> |
|
53024 | 74 |
G \<turnstile> (None, hp0, (stk0,lvars0,C,S, pc0)#frs) \<midarrow>jvm\<rightarrow> |
13673 | 75 |
(None, hp1, (stk1,lvars1,C,S, Suc pc0)#frs)" |
76 |
apply (unfold exec_all_def) |
|
77 |
apply (rule r_into_rtrancl) |
|
78 |
apply (simp add: gis_def gmb_def split_beta) |
|
79 |
done |
|
80 |
||
81 |
||
82 |
(***********************************************************************) |
|
83 |
||
35416
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
haftmann
parents:
33639
diff
changeset
|
84 |
definition progression :: "jvm_prog \<Rightarrow> cname \<Rightarrow> sig \<Rightarrow> |
13673 | 85 |
aheap \<Rightarrow> opstack \<Rightarrow> locvars \<Rightarrow> |
86 |
bytecode \<Rightarrow> |
|
87 |
aheap \<Rightarrow> opstack \<Rightarrow> locvars \<Rightarrow> |
|
88 |
bool" |
|
35416
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
haftmann
parents:
33639
diff
changeset
|
89 |
("{_,_,_} \<turnstile> {_, _, _} >- _ \<rightarrow> {_, _, _}" [61,61,61,61,61,61,90,61,61,61]60) where |
13673 | 90 |
"{G,C,S} \<turnstile> {hp0, os0, lvars0} >- instrs \<rightarrow> {hp1, os1, lvars1} == |
91 |
\<forall> pre post frs. |
|
92 |
(gis (gmb G C S) = pre @ instrs @ post) \<longrightarrow> |
|
53024 | 93 |
G \<turnstile> (None,hp0,(os0,lvars0,C,S,length pre)#frs) \<midarrow>jvm\<rightarrow> |
13673 | 94 |
(None,hp1,(os1,lvars1,C,S,(length pre) + (length instrs))#frs)" |
95 |
||
96 |
||
97 |
||
98 |
lemma progression_call: |
|
99 |
"\<lbrakk> \<forall> pc frs. |
|
100 |
exec_instr instr G hp0 os0 lvars0 C S pc frs = |
|
101 |
(None, hp', (os', lvars', C', S', 0) # (fr pc) # frs) \<and> |
|
102 |
gis (gmb G C' S') = instrs' @ [Return] \<and> |
|
103 |
{G, C', S'} \<turnstile> {hp', os', lvars'} >- instrs' \<rightarrow> {hp'', os'', lvars''} \<and> |
|
104 |
exec_instr Return G hp'' os'' lvars'' C' S' (length instrs') |
|
105 |
((fr pc) # frs) = |
|
106 |
(None, hp2, (os2, lvars2, C, S, Suc pc) # frs) \<rbrakk> \<Longrightarrow> |
|
107 |
{G, C, S} \<turnstile> {hp0, os0, lvars0} >-[instr]\<rightarrow> {hp2,os2,lvars2}" |
|
108 |
apply (simp only: progression_def) |
|
109 |
apply (intro strip) |
|
110 |
apply (drule_tac x="length pre" in spec) |
|
111 |
apply (drule_tac x="frs" in spec) |
|
112 |
apply clarify |
|
113 |
apply (rule exec_all_trans) |
|
114 |
apply (rule exec_instr_in_exec_all) apply simp |
|
115 |
apply simp |
|
116 |
apply (rule exec_all_trans) |
|
117 |
apply (simp only: append_Nil) |
|
118 |
apply (drule_tac x="[]" in spec) |
|
24699
c6674504103f
datatype interpretators for size and datatype_realizer
haftmann
parents:
24074
diff
changeset
|
119 |
apply (simp only: list.simps list.size) |
13673 | 120 |
apply blast |
121 |
apply (rule exec_instr_in_exec_all) |
|
122 |
apply auto |
|
123 |
done |
|
124 |
||
125 |
||
126 |
lemma progression_transitive: |
|
127 |
"\<lbrakk> instrs_comb = instrs0 @ instrs1; |
|
128 |
{G, C, S} \<turnstile> {hp0, os0, lvars0} >- instrs0 \<rightarrow> {hp1, os1, lvars1}; |
|
129 |
{G, C, S} \<turnstile> {hp1, os1, lvars1} >- instrs1 \<rightarrow> {hp2, os2, lvars2} \<rbrakk> |
|
130 |
\<Longrightarrow> |
|
131 |
{G, C, S} \<turnstile> {hp0, os0, lvars0} >- instrs_comb \<rightarrow> {hp2, os2, lvars2}" |
|
132 |
apply (simp only: progression_def) |
|
133 |
apply (intro strip) |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
134 |
apply (rule_tac ?s1.0 = "Norm (hp1, (os1, lvars1, C, S, |
13673 | 135 |
length pre + length instrs0) # frs)" |
136 |
in exec_all_trans) |
|
137 |
apply (simp only: append_assoc) |
|
138 |
apply (erule thin_rl, erule thin_rl) |
|
139 |
apply (drule_tac x="pre @ instrs0" in spec) |
|
140 |
apply (simp add: add_assoc) |
|
141 |
done |
|
142 |
||
143 |
lemma progression_refl: |
|
144 |
"{G, C, S} \<turnstile> {hp0, os0, lvars0} >- [] \<rightarrow> {hp0, os0, lvars0}" |
|
145 |
apply (simp add: progression_def) |
|
146 |
apply (intro strip) |
|
147 |
apply (rule exec_all_refl) |
|
148 |
done |
|
149 |
||
150 |
lemma progression_one_step: " |
|
151 |
\<forall> pc frs. |
|
152 |
(exec_instr i G hp0 os0 lvars0 C S pc frs) = |
|
153 |
(None, hp1, (os1,lvars1,C,S, Suc pc)#frs) |
|
154 |
\<Longrightarrow> {G, C, S} \<turnstile> {hp0, os0, lvars0} >- [i] \<rightarrow> {hp1, os1, lvars1}" |
|
155 |
apply (unfold progression_def) |
|
156 |
apply (intro strip) |
|
157 |
apply simp |
|
158 |
apply (rule exec_all_one_step) |
|
159 |
apply auto |
|
160 |
done |
|
161 |
||
162 |
(*****) |
|
35416
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
haftmann
parents:
33639
diff
changeset
|
163 |
definition jump_fwd :: "jvm_prog \<Rightarrow> cname \<Rightarrow> sig \<Rightarrow> |
13673 | 164 |
aheap \<Rightarrow> locvars \<Rightarrow> opstack \<Rightarrow> opstack \<Rightarrow> |
35416
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
haftmann
parents:
33639
diff
changeset
|
165 |
instr \<Rightarrow> bytecode \<Rightarrow> bool" where |
13673 | 166 |
"jump_fwd G C S hp lvars os0 os1 instr instrs == |
167 |
\<forall> pre post frs. |
|
168 |
(gis (gmb G C S) = pre @ instr # instrs @ post) \<longrightarrow> |
|
169 |
exec_all G (None,hp,(os0,lvars,C,S, length pre)#frs) |
|
170 |
(None,hp,(os1,lvars,C,S,(length pre) + (length instrs) + 1)#frs)" |
|
171 |
||
172 |
||
173 |
lemma jump_fwd_one_step: |
|
174 |
"\<forall> pc frs. |
|
175 |
exec_instr instr G hp os0 lvars C S pc frs = |
|
176 |
(None, hp, (os1, lvars, C, S, pc + (length instrs) + 1)#frs) |
|
177 |
\<Longrightarrow> jump_fwd G C S hp lvars os0 os1 instr instrs" |
|
178 |
apply (unfold jump_fwd_def) |
|
179 |
apply (intro strip) |
|
180 |
apply (rule exec_instr_in_exec_all) |
|
181 |
apply auto |
|
182 |
done |
|
183 |
||
184 |
||
185 |
lemma jump_fwd_progression_aux: |
|
186 |
"\<lbrakk> instrs_comb = instr # instrs0 @ instrs1; |
|
187 |
jump_fwd G C S hp lvars os0 os1 instr instrs0; |
|
188 |
{G, C, S} \<turnstile> {hp, os1, lvars} >- instrs1 \<rightarrow> {hp2, os2, lvars2} \<rbrakk> |
|
189 |
\<Longrightarrow> {G, C, S} \<turnstile> {hp, os0, lvars} >- instrs_comb \<rightarrow> {hp2, os2, lvars2}" |
|
190 |
apply (simp only: progression_def jump_fwd_def) |
|
191 |
apply (intro strip) |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
192 |
apply (rule_tac ?s1.0 = "Norm(hp, (os1, lvars, C, S, length pre + length instrs0 + 1) # frs)" in exec_all_trans) |
13673 | 193 |
apply (simp only: append_assoc) |
194 |
apply (subgoal_tac "pre @ (instr # instrs0 @ instrs1) @ post = pre @ instr # instrs0 @ (instrs1 @ post)") |
|
195 |
apply blast |
|
196 |
apply simp |
|
197 |
apply (erule thin_rl, erule thin_rl) |
|
198 |
apply (drule_tac x="pre @ instr # instrs0" in spec) |
|
199 |
apply (simp add: add_assoc) |
|
200 |
done |
|
201 |
||
202 |
||
203 |
lemma jump_fwd_progression: |
|
204 |
"\<lbrakk> instrs_comb = instr # instrs0 @ instrs1; |
|
205 |
\<forall> pc frs. |
|
206 |
exec_instr instr G hp os0 lvars C S pc frs = |
|
207 |
(None, hp, (os1, lvars, C, S, pc + (length instrs0) + 1)#frs); |
|
208 |
{G, C, S} \<turnstile> {hp, os1, lvars} >- instrs1 \<rightarrow> {hp2, os2, lvars2} \<rbrakk> |
|
209 |
\<Longrightarrow> {G, C, S} \<turnstile> {hp, os0, lvars} >- instrs_comb \<rightarrow> {hp2, os2, lvars2}" |
|
210 |
apply (rule jump_fwd_progression_aux) |
|
211 |
apply assumption |
|
212 |
apply (rule jump_fwd_one_step) apply assumption+ |
|
213 |
done |
|
214 |
||
215 |
||
216 |
(* note: instrs and instr reversed wrt. jump_fwd *) |
|
35416
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
haftmann
parents:
33639
diff
changeset
|
217 |
definition jump_bwd :: "jvm_prog \<Rightarrow> cname \<Rightarrow> sig \<Rightarrow> |
13673 | 218 |
aheap \<Rightarrow> locvars \<Rightarrow> opstack \<Rightarrow> opstack \<Rightarrow> |
35416
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
haftmann
parents:
33639
diff
changeset
|
219 |
bytecode \<Rightarrow> instr \<Rightarrow> bool" where |
13673 | 220 |
"jump_bwd G C S hp lvars os0 os1 instrs instr == |
221 |
\<forall> pre post frs. |
|
222 |
(gis (gmb G C S) = pre @ instrs @ instr # post) \<longrightarrow> |
|
223 |
exec_all G (None,hp,(os0,lvars,C,S, (length pre) + (length instrs))#frs) |
|
224 |
(None,hp,(os1,lvars,C,S, (length pre))#frs)" |
|
225 |
||
226 |
||
227 |
lemma jump_bwd_one_step: |
|
228 |
"\<forall> pc frs. |
|
229 |
exec_instr instr G hp os0 lvars C S (pc + (length instrs)) frs = |
|
230 |
(None, hp, (os1, lvars, C, S, pc)#frs) |
|
231 |
\<Longrightarrow> |
|
232 |
jump_bwd G C S hp lvars os0 os1 instrs instr" |
|
233 |
apply (unfold jump_bwd_def) |
|
234 |
apply (intro strip) |
|
235 |
apply (rule exec_instr_in_exec_all) |
|
236 |
apply auto |
|
237 |
done |
|
238 |
||
239 |
lemma jump_bwd_progression: |
|
240 |
"\<lbrakk> instrs_comb = instrs @ [instr]; |
|
241 |
{G, C, S} \<turnstile> {hp0, os0, lvars0} >- instrs \<rightarrow> {hp1, os1, lvars1}; |
|
242 |
jump_bwd G C S hp1 lvars1 os1 os2 instrs instr; |
|
243 |
{G, C, S} \<turnstile> {hp1, os2, lvars1} >- instrs_comb \<rightarrow> {hp3, os3, lvars3} \<rbrakk> |
|
244 |
\<Longrightarrow> {G, C, S} \<turnstile> {hp0, os0, lvars0} >- instrs_comb \<rightarrow> {hp3, os3, lvars3}" |
|
245 |
apply (simp only: progression_def jump_bwd_def) |
|
246 |
apply (intro strip) |
|
247 |
apply (rule exec_all_trans, force) |
|
248 |
apply (rule exec_all_trans, force) |
|
249 |
apply (rule exec_all_trans, force) |
|
250 |
apply simp |
|
251 |
apply (rule exec_all_refl) |
|
252 |
done |
|
253 |
||
254 |
||
255 |
(**********************************************************************) |
|
256 |
||
257 |
(* class C with signature S is defined in program G *) |
|
35416
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
haftmann
parents:
33639
diff
changeset
|
258 |
definition class_sig_defined :: "'c prog \<Rightarrow> cname \<Rightarrow> sig \<Rightarrow> bool" where |
13673 | 259 |
"class_sig_defined G C S == |
260 |
is_class G C \<and> (\<exists> D rT mb. (method (G, C) S = Some (D, rT, mb)))" |
|
261 |
||
262 |
||
263 |
(* The environment of a java method body |
|
264 |
(characterized by class and signature) *) |
|
35416
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
haftmann
parents:
33639
diff
changeset
|
265 |
definition env_of_jmb :: "java_mb prog \<Rightarrow> cname \<Rightarrow> sig \<Rightarrow> java_mb env" where |
13673 | 266 |
"env_of_jmb G C S == |
267 |
(let (mn,pTs) = S; |
|
268 |
(D,rT,(pns,lvars,blk,res)) = the(method (G, C) S) in |
|
269 |
(G,map_of lvars(pns[\<mapsto>]pTs)(This\<mapsto>Class C)))" |
|
270 |
||
271 |
lemma env_of_jmb_fst [simp]: "fst (env_of_jmb G C S) = G" |
|
272 |
by (simp add: env_of_jmb_def split_beta) |
|
273 |
||
274 |
||
275 |
(**********************************************************************) |
|
276 |
||
277 |
||
278 |
lemma method_preserves [rule_format (no_asm)]: |
|
279 |
"\<lbrakk> wf_prog wf_mb G; is_class G C; |
|
280 |
\<forall> S rT mb. \<forall> cn \<in> fst ` set G. wf_mdecl wf_mb G cn (S,rT,mb) \<longrightarrow> (P cn S (rT,mb))\<rbrakk> |
|
281 |
\<Longrightarrow> \<forall> D. |
|
282 |
method (G, C) S = Some (D, rT, mb) \<longrightarrow> (P D S (rT,mb))" |
|
283 |
||
14045 | 284 |
apply (frule wf_prog_ws_prog [THEN wf_subcls1]) |
13673 | 285 |
apply (rule subcls1_induct, assumption, assumption) |
286 |
||
287 |
apply (intro strip) |
|
288 |
apply ((drule spec)+, drule_tac x="Object" in bspec) |
|
14045 | 289 |
apply (simp add: wf_prog_def ws_prog_def wf_syscls_def) |
13673 | 290 |
apply (subgoal_tac "D=Object") apply simp |
291 |
apply (drule mp) |
|
292 |
apply (frule_tac C=Object in method_wf_mdecl) |
|
14045 | 293 |
apply simp |
294 |
apply assumption apply simp apply assumption apply simp |
|
13673 | 295 |
|
15481 | 296 |
apply (simplesubst method_rec) apply simp |
13673 | 297 |
apply force |
14045 | 298 |
apply simp |
14025 | 299 |
apply (simp only: map_add_def) |
13673 | 300 |
apply (split option.split) |
301 |
apply (rule conjI) |
|
302 |
apply force |
|
303 |
apply (intro strip) |
|
304 |
apply (frule_tac |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
305 |
?P1.0 = "wf_mdecl wf_mb G Ca" and |
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
306 |
?P2.0 = "%(S, (Da, rT, mb)). P Da S (rT, mb)" in map_of_map_prop) |
13673 | 307 |
apply (force simp: wf_cdecl_def) |
308 |
||
309 |
apply clarify |
|
310 |
||
311 |
apply (simp only: class_def) |
|
312 |
apply (drule map_of_SomeD)+ |
|
313 |
apply (frule_tac A="set G" and f=fst in imageI, simp) |
|
314 |
apply blast |
|
315 |
apply simp |
|
316 |
done |
|
317 |
||
318 |
||
319 |
lemma method_preserves_length: |
|
320 |
"\<lbrakk> wf_java_prog G; is_class G C; |
|
321 |
method (G, C) (mn,pTs) = Some (D, rT, pns, lvars, blk, res)\<rbrakk> |
|
322 |
\<Longrightarrow> length pns = length pTs" |
|
323 |
apply (frule_tac |
|
324 |
P="%D (mn,pTs) (rT, pns, lvars, blk, res). length pns = length pTs" |
|
325 |
in method_preserves) |
|
326 |
apply (auto simp: wf_mdecl_def wf_java_mdecl_def) |
|
327 |
done |
|
328 |
||
329 |
(**********************************************************************) |
|
330 |
||
35416
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
haftmann
parents:
33639
diff
changeset
|
331 |
definition wtpd_expr :: "java_mb env \<Rightarrow> expr \<Rightarrow> bool" where |
13673 | 332 |
"wtpd_expr E e == (\<exists> T. E\<turnstile>e :: T)" |
35416
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
haftmann
parents:
33639
diff
changeset
|
333 |
|
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
haftmann
parents:
33639
diff
changeset
|
334 |
definition wtpd_exprs :: "java_mb env \<Rightarrow> (expr list) \<Rightarrow> bool" where |
13673 | 335 |
"wtpd_exprs E e == (\<exists> T. E\<turnstile>e [::] T)" |
35416
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
haftmann
parents:
33639
diff
changeset
|
336 |
|
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
haftmann
parents:
33639
diff
changeset
|
337 |
definition wtpd_stmt :: "java_mb env \<Rightarrow> stmt \<Rightarrow> bool" where |
13673 | 338 |
"wtpd_stmt E c == (E\<turnstile>c \<surd>)" |
339 |
||
340 |
lemma wtpd_expr_newc: "wtpd_expr E (NewC C) \<Longrightarrow> is_class (prg E) C" |
|
341 |
by (simp only: wtpd_expr_def, erule exE, erule ty_expr.cases, auto) |
|
342 |
||
343 |
lemma wtpd_expr_cast: "wtpd_expr E (Cast cn e) \<Longrightarrow> (wtpd_expr E e)" |
|
344 |
by (simp only: wtpd_expr_def, erule exE, erule ty_expr.cases, auto) |
|
345 |
||
346 |
lemma wtpd_expr_lacc: "\<lbrakk> wtpd_expr (env_of_jmb G C S) (LAcc vn); |
|
347 |
class_sig_defined G C S \<rbrakk> |
|
348 |
\<Longrightarrow> vn \<in> set (gjmb_plns (gmb G C S)) \<or> vn = This" |
|
349 |
apply (simp only: wtpd_expr_def env_of_jmb_def class_sig_defined_def galldefs) |
|
350 |
apply clarify |
|
351 |
apply (case_tac S) |
|
352 |
apply simp |
|
353 |
apply (erule ty_expr.cases) |
|
354 |
apply (auto dest: map_upds_SomeD map_of_SomeD fst_in_set_lemma) |
|
355 |
apply (drule map_upds_SomeD) |
|
356 |
apply (erule disjE) |
|
357 |
apply assumption |
|
358 |
apply (drule map_of_SomeD) apply (auto dest: fst_in_set_lemma) |
|
359 |
done |
|
360 |
||
361 |
lemma wtpd_expr_lass: "wtpd_expr E (vn::=e) |
|
362 |
\<Longrightarrow> (vn \<noteq> This) & (wtpd_expr E (LAcc vn)) & (wtpd_expr E e)" |
|
363 |
by (simp only: wtpd_expr_def, erule exE, erule ty_expr.cases, auto) |
|
364 |
||
365 |
lemma wtpd_expr_facc: "wtpd_expr E ({fd}a..fn) |
|
366 |
\<Longrightarrow> (wtpd_expr E a)" |
|
367 |
by (simp only: wtpd_expr_def, erule exE, erule ty_expr.cases, auto) |
|
368 |
||
369 |
lemma wtpd_expr_fass: "wtpd_expr E ({fd}a..fn:=v) |
|
370 |
\<Longrightarrow> (wtpd_expr E ({fd}a..fn)) & (wtpd_expr E v)" |
|
371 |
by (simp only: wtpd_expr_def, erule exE, erule ty_expr.cases, auto) |
|
372 |
||
373 |
||
374 |
lemma wtpd_expr_binop: "wtpd_expr E (BinOp bop e1 e2) |
|
375 |
\<Longrightarrow> (wtpd_expr E e1) & (wtpd_expr E e2)" |
|
376 |
by (simp only: wtpd_expr_def, erule exE, erule ty_expr.cases, auto) |
|
377 |
||
378 |
lemma wtpd_exprs_cons: "wtpd_exprs E (e # es) |
|
379 |
\<Longrightarrow> (wtpd_expr E e) & (wtpd_exprs E es)" |
|
380 |
by (simp only: wtpd_exprs_def wtpd_expr_def, erule exE, erule ty_exprs.cases, auto) |
|
381 |
||
382 |
lemma wtpd_stmt_expr: "wtpd_stmt E (Expr e) \<Longrightarrow> (wtpd_expr E e)" |
|
383 |
by (simp only: wtpd_stmt_def wtpd_expr_def, erule wt_stmt.cases, auto) |
|
384 |
||
385 |
lemma wtpd_stmt_comp: "wtpd_stmt E (s1;; s2) \<Longrightarrow> |
|
386 |
(wtpd_stmt E s1) & (wtpd_stmt E s2)" |
|
387 |
by (simp only: wtpd_stmt_def wtpd_expr_def, erule wt_stmt.cases, auto) |
|
388 |
||
389 |
lemma wtpd_stmt_cond: "wtpd_stmt E (If(e) s1 Else s2) \<Longrightarrow> |
|
390 |
(wtpd_expr E e) & (wtpd_stmt E s1) & (wtpd_stmt E s2) |
|
391 |
& (E\<turnstile>e::PrimT Boolean)" |
|
392 |
by (simp only: wtpd_stmt_def wtpd_expr_def, erule wt_stmt.cases, auto) |
|
393 |
||
394 |
lemma wtpd_stmt_loop: "wtpd_stmt E (While(e) s) \<Longrightarrow> |
|
395 |
(wtpd_expr E e) & (wtpd_stmt E s) & (E\<turnstile>e::PrimT Boolean)" |
|
396 |
by (simp only: wtpd_stmt_def wtpd_expr_def, erule wt_stmt.cases, auto) |
|
397 |
||
398 |
lemma wtpd_expr_call: "wtpd_expr E ({C}a..mn({pTs'}ps)) |
|
399 |
\<Longrightarrow> (wtpd_expr E a) & (wtpd_exprs E ps) |
|
400 |
& (length ps = length pTs') & (E\<turnstile>a::Class C) |
|
401 |
& (\<exists> pTs md rT. |
|
402 |
E\<turnstile>ps[::]pTs & max_spec (prg E) C (mn, pTs) = {((md,rT),pTs')})" |
|
403 |
apply (simp only: wtpd_expr_def wtpd_exprs_def) |
|
404 |
apply (erule exE) |
|
23757 | 405 |
apply (ind_cases "E \<turnstile> {C}a..mn( {pTs'}ps) :: T" for T) |
13673 | 406 |
apply (auto simp: max_spec_preserves_length) |
407 |
done |
|
408 |
||
409 |
lemma wtpd_blk: |
|
410 |
"\<lbrakk> method (G, D) (md, pTs) = Some (D, rT, (pns, lvars, blk, res)); |
|
411 |
wf_prog wf_java_mdecl G; is_class G D \<rbrakk> |
|
412 |
\<Longrightarrow> wtpd_stmt (env_of_jmb G D (md, pTs)) blk" |
|
413 |
apply (simp add: wtpd_stmt_def env_of_jmb_def) |
|
414 |
apply (frule_tac P="%D (md, pTs) (rT, (pns, lvars, blk, res)). (G, map_of lvars(pns[\<mapsto>]pTs)(This\<mapsto>Class D)) \<turnstile> blk \<surd> " in method_preserves) |
|
415 |
apply (auto simp: wf_mdecl_def wf_java_mdecl_def) |
|
416 |
done |
|
417 |
||
418 |
lemma wtpd_res: |
|
419 |
"\<lbrakk> method (G, D) (md, pTs) = Some (D, rT, (pns, lvars, blk, res)); |
|
420 |
wf_prog wf_java_mdecl G; is_class G D \<rbrakk> |
|
421 |
\<Longrightarrow> wtpd_expr (env_of_jmb G D (md, pTs)) res" |
|
422 |
apply (simp add: wtpd_expr_def env_of_jmb_def) |
|
423 |
apply (frule_tac P="%D (md, pTs) (rT, (pns, lvars, blk, res)). \<exists>T. (G, map_of lvars(pns[\<mapsto>]pTs)(This\<mapsto>Class D)) \<turnstile> res :: T " in method_preserves) |
|
424 |
apply (auto simp: wf_mdecl_def wf_java_mdecl_def) |
|
425 |
done |
|
426 |
||
427 |
||
428 |
(**********************************************************************) |
|
429 |
||
430 |
||
431 |
(* Is there a more elegant proof? *) |
|
432 |
lemma evals_preserves_length: |
|
433 |
"G\<turnstile> xs -es[\<succ>]vs-> (None, s) \<Longrightarrow> length es = length vs" |
|
434 |
apply (subgoal_tac |
|
435 |
"\<forall> xs'. (G \<turnstile> xk -xj\<succ>xi-> xh \<longrightarrow> True) & |
|
436 |
(G\<turnstile> xs -es[\<succ>]vs-> xs' \<longrightarrow> (\<exists> s. (xs' = (None, s))) \<longrightarrow> |
|
437 |
length es = length vs) & |
|
22271 | 438 |
(G \<turnstile> xc -xb-> xa \<longrightarrow> True)") |
13673 | 439 |
apply blast |
440 |
apply (rule allI) |
|
441 |
apply (rule Eval.eval_evals_exec.induct) |
|
442 |
apply auto |
|
443 |
done |
|
444 |
||
445 |
(***********************************************************************) |
|
446 |
||
447 |
(* required for translation of BinOp *) |
|
448 |
||
449 |
||
450 |
lemma progression_Eq : "{G, C, S} \<turnstile> |
|
451 |
{hp, (v2 # v1 # os), lvars} |
|
452 |
>- [Ifcmpeq 3, LitPush (Bool False), Goto 2, LitPush (Bool True)] \<rightarrow> |
|
453 |
{hp, (Bool (v1 = v2) # os), lvars}" |
|
454 |
apply (case_tac "v1 = v2") |
|
455 |
||
456 |
(* case v1 = v2 *) |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
457 |
apply (rule_tac ?instrs1.0 = "[LitPush (Bool True)]" in jump_fwd_progression) |
13837
8dd150d36c65
Reorganized, moving many results about the integer dvd relation from IntPrimes
paulson
parents:
13673
diff
changeset
|
458 |
apply (auto simp: nat_add_distrib) |
13673 | 459 |
apply (rule progression_one_step) apply simp |
460 |
||
461 |
(* case v1 \<noteq> v2 *) |
|
462 |
apply (rule progression_one_step [THEN HOL.refl [THEN progression_transitive], simplified]) |
|
463 |
apply auto |
|
464 |
apply (rule progression_one_step [THEN HOL.refl [THEN progression_transitive], simplified]) |
|
465 |
apply auto |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
466 |
apply (rule_tac ?instrs1.0 = "[]" in jump_fwd_progression) |
13837
8dd150d36c65
Reorganized, moving many results about the integer dvd relation from IntPrimes
paulson
parents:
13673
diff
changeset
|
467 |
apply (auto simp: nat_add_distrib intro: progression_refl) |
13673 | 468 |
done |
469 |
||
470 |
||
471 |
(**********************************************************************) |
|
472 |
||
473 |
||
474 |
(* to avoid automatic pair splits *) |
|
475 |
||
476 |
declare split_paired_All [simp del] split_paired_Ex [simp del] |
|
477 |
||
478 |
lemma distinct_method: "\<lbrakk> wf_java_prog G; is_class G C; |
|
479 |
method (G, C) S = Some (D, rT, pns, lvars, blk, res) \<rbrakk> \<Longrightarrow> |
|
480 |
distinct (gjmb_plns (gmb G C S))" |
|
481 |
apply (frule method_wf_mdecl [THEN conjunct2], assumption, assumption) |
|
482 |
apply (case_tac S) |
|
46226 | 483 |
apply (simp add: wf_mdecl_def wf_java_mdecl_def galldefs) |
13673 | 484 |
apply (simp add: unique_def map_of_in_set) |
485 |
apply blast |
|
486 |
done |
|
487 |
||
488 |
lemma distinct_method_if_class_sig_defined : |
|
489 |
"\<lbrakk> wf_java_prog G; class_sig_defined G C S \<rbrakk> \<Longrightarrow> |
|
490 |
distinct (gjmb_plns (gmb G C S))" |
|
491 |
by (auto intro: distinct_method simp: class_sig_defined_def) |
|
492 |
||
493 |
||
494 |
lemma method_yields_wf_java_mdecl: "\<lbrakk> wf_java_prog G; is_class G C; |
|
495 |
method (G, C) S = Some (D, rT, pns, lvars, blk, res) \<rbrakk> \<Longrightarrow> |
|
496 |
wf_java_mdecl G D (S,rT,(pns,lvars,blk,res))" |
|
497 |
apply (frule method_wf_mdecl) |
|
498 |
apply (auto simp: wf_mdecl_def) |
|
499 |
done |
|
500 |
||
501 |
(**********************************************************************) |
|
502 |
||
503 |
||
504 |
lemma progression_lvar_init_aux [rule_format (no_asm)]: " |
|
505 |
\<forall> zs prfx lvals lvars0. |
|
506 |
lvars0 = (zs @ lvars) \<longrightarrow> |
|
507 |
(disjoint_varnames pns lvars0 \<longrightarrow> |
|
508 |
(length lvars = length lvals) \<longrightarrow> |
|
509 |
(Suc(length pns + length zs) = length prfx) \<longrightarrow> |
|
510 |
({cG, D, S} \<turnstile> |
|
511 |
{h, os, (prfx @ lvals)} |
|
512 |
>- (concat (map (compInit (pns, lvars0, blk, res)) lvars)) \<rightarrow> |
|
513 |
{h, os, (prfx @ (map (\<lambda>p. (default_val (snd p))) lvars))}))" |
|
514 |
apply simp |
|
515 |
apply (induct lvars) |
|
516 |
apply (clarsimp, rule progression_refl) |
|
517 |
apply (intro strip) |
|
518 |
apply (case_tac lvals) apply simp |
|
519 |
apply (simp (no_asm_simp) ) |
|
520 |
||
15236
f289e8ba2bb3
Proofs needed to be updated because induction now preserves name of
nipkow
parents:
15097
diff
changeset
|
521 |
apply (rule_tac ?lvars1.0 = "(prfx @ [default_val (snd a)]) @ list" in progression_transitive, rule HOL.refl) |
13673 | 522 |
apply (case_tac a) apply (simp (no_asm_simp) add: compInit_def) |
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
523 |
apply (rule_tac ?instrs0.0 = "[load_default_val b]" in progression_transitive, simp) |
13673 | 524 |
apply (rule progression_one_step) |
525 |
apply (simp (no_asm_simp) add: load_default_val_def) |
|
526 |
apply (rule conjI, simp)+ apply (rule HOL.refl) |
|
527 |
||
528 |
apply (rule progression_one_step) |
|
529 |
apply (simp (no_asm_simp)) |
|
530 |
apply (rule conjI, simp)+ |
|
531 |
apply (simp add: index_of_var2) |
|
532 |
apply (drule_tac x="zs @ [a]" in spec) (* instantiate zs *) |
|
533 |
apply (drule mp, simp) |
|
534 |
apply (drule_tac x="(prfx @ [default_val (snd a)])" in spec) (* instantiate prfx *) |
|
535 |
apply auto |
|
536 |
done |
|
537 |
||
538 |
lemma progression_lvar_init [rule_format (no_asm)]: |
|
539 |
"\<lbrakk> wf_java_prog G; is_class G C; |
|
540 |
method (G, C) S = Some (D, rT, pns, lvars, blk, res) \<rbrakk> \<Longrightarrow> |
|
541 |
length pns = length pvs \<longrightarrow> |
|
542 |
(\<forall> lvals. |
|
543 |
length lvars = length lvals \<longrightarrow> |
|
544 |
{cG, D, S} \<turnstile> |
|
545 |
{h, os, (a' # pvs @ lvals)} |
|
546 |
>- (compInitLvars (pns, lvars, blk, res) lvars) \<rightarrow> |
|
547 |
{h, os, (locvars_xstate G C S (Norm (h, init_vars lvars(pns[\<mapsto>]pvs)(This\<mapsto>a'))))})" |
|
548 |
apply (simp only: compInitLvars_def) |
|
549 |
apply (frule method_yields_wf_java_mdecl, assumption, assumption) |
|
550 |
||
551 |
apply (simp only: wf_java_mdecl_def) |
|
552 |
apply (subgoal_tac "(\<forall>y\<in>set pns. y \<notin> set (map fst lvars))") |
|
33639
603320b93668
New list theorems; added map_map to simpset, this is the prefered direction; allow sorting by a key
hoelzl
parents:
32960
diff
changeset
|
553 |
apply (simp add: init_vars_def locvars_xstate_def locvars_locals_def galldefs unique_def split_def map_of_map_as_map_upd del: map_map) |
13673 | 554 |
apply (intro strip) |
555 |
apply (simp (no_asm_simp) only: append_Cons [THEN sym]) |
|
556 |
apply (rule progression_lvar_init_aux) |
|
557 |
apply (auto simp: unique_def map_of_in_set disjoint_varnames_def) |
|
558 |
done |
|
559 |
||
560 |
||
561 |
||
562 |
||
563 |
(**********************************************************************) |
|
564 |
||
14045 | 565 |
lemma state_ok_eval: "\<lbrakk>xs::\<preceq>E; wf_java_prog (prg E); wtpd_expr E e; |
566 |
(prg E)\<turnstile>xs -e\<succ>v -> xs'\<rbrakk> \<Longrightarrow> xs'::\<preceq>E" |
|
567 |
apply (simp only: wtpd_expr_def) |
|
13673 | 568 |
apply (erule exE) |
14045 | 569 |
apply (case_tac xs', case_tac xs) |
570 |
apply (auto intro: eval_type_sound [THEN conjunct1]) |
|
13673 | 571 |
done |
572 |
||
14045 | 573 |
lemma state_ok_evals: "\<lbrakk>xs::\<preceq>E; wf_java_prog (prg E); wtpd_exprs E es; |
22271 | 574 |
prg E \<turnstile> xs -es[\<succ>]vs-> xs'\<rbrakk> \<Longrightarrow> xs'::\<preceq>E" |
14045 | 575 |
apply (simp only: wtpd_exprs_def) |
576 |
apply (erule exE) |
|
577 |
apply (case_tac xs) apply (case_tac xs') |
|
578 |
apply (auto intro: evals_type_sound [THEN conjunct1]) |
|
13673 | 579 |
done |
580 |
||
14045 | 581 |
lemma state_ok_exec: "\<lbrakk>xs::\<preceq>E; wf_java_prog (prg E); wtpd_stmt E st; |
22271 | 582 |
prg E \<turnstile> xs -st-> xs'\<rbrakk> \<Longrightarrow> xs'::\<preceq>E" |
14045 | 583 |
apply (simp only: wtpd_stmt_def) |
584 |
apply (case_tac xs', case_tac xs) |
|
14143 | 585 |
apply (auto dest: exec_type_sound) |
13673 | 586 |
done |
587 |
||
588 |
||
589 |
lemma state_ok_init: |
|
14045 | 590 |
"\<lbrakk> wf_java_prog G; (x, h, l)::\<preceq>(env_of_jmb G C S); |
13673 | 591 |
is_class G dynT; |
592 |
method (G, dynT) (mn, pTs) = Some (md, rT, pns, lvars, blk, res); |
|
593 |
list_all2 (conf G h) pvs pTs; G,h \<turnstile> a' ::\<preceq> Class md\<rbrakk> |
|
594 |
\<Longrightarrow> |
|
14045 | 595 |
(np a' x, h, init_vars lvars(pns[\<mapsto>]pvs)(This\<mapsto>a'))::\<preceq>(env_of_jmb G md (mn, pTs))" |
596 |
apply (frule wf_prog_ws_prog) |
|
13673 | 597 |
apply (frule method_in_md [THEN conjunct2], assumption+) |
598 |
apply (frule method_yields_wf_java_mdecl, assumption, assumption) |
|
14045 | 599 |
apply (simp add: env_of_jmb_def gs_def conforms_def split_beta) |
13673 | 600 |
apply (simp add: wf_java_mdecl_def) |
601 |
apply (rule conjI) |
|
602 |
apply (rule lconf_ext) |
|
603 |
apply (rule lconf_ext_list) |
|
604 |
apply (rule lconf_init_vars) |
|
605 |
apply (auto dest: Ball_set_table) |
|
606 |
apply (simp add: np_def xconf_raise_if) |
|
607 |
done |
|
608 |
||
609 |
||
610 |
lemma ty_exprs_list_all2 [rule_format (no_asm)]: |
|
611 |
"(\<forall> Ts. (E \<turnstile> es [::] Ts) = list_all2 (\<lambda>e T. E \<turnstile> e :: T) es Ts)" |
|
612 |
apply (rule list.induct) |
|
613 |
apply simp |
|
614 |
apply (rule allI) |
|
615 |
apply (rule iffI) |
|
23757 | 616 |
apply (ind_cases "E \<turnstile> [] [::] Ts" for Ts, assumption) |
13673 | 617 |
apply simp apply (rule WellType.Nil) |
618 |
apply (simp add: list_all2_Cons1) |
|
619 |
apply (rule allI) |
|
620 |
apply (rule iffI) |
|
621 |
apply (rename_tac a exs Ts) |
|
23757 | 622 |
apply (ind_cases "E \<turnstile> a # exs [::] Ts" for a exs Ts) apply blast |
13673 | 623 |
apply (auto intro: WellType.Cons) |
624 |
done |
|
625 |
||
626 |
||
627 |
lemma conf_bool: "G,h \<turnstile> v::\<preceq>PrimT Boolean \<Longrightarrow> \<exists> b. v = Bool b" |
|
628 |
apply (simp add: conf_def) |
|
629 |
apply (erule exE) |
|
630 |
apply (case_tac v) |
|
631 |
apply (auto elim: widen.cases) |
|
632 |
done |
|
633 |
||
634 |
||
14045 | 635 |
lemma class_expr_is_class: "\<lbrakk>E \<turnstile> e :: Class C; ws_prog (prg E)\<rbrakk> |
13673 | 636 |
\<Longrightarrow> is_class (prg E) C" |
637 |
by (case_tac E, auto dest: ty_expr_is_type) |
|
638 |
||
639 |
||
640 |
lemma max_spec_widen: "max_spec G C (mn, pTs) = {((md,rT),pTs')} \<Longrightarrow> |
|
641 |
list_all2 (\<lambda> T T'. G \<turnstile> T \<preceq> T') pTs pTs'" |
|
642 |
by (blast dest: singleton_in_set max_spec2appl_meths appl_methsD) |
|
643 |
||
644 |
||
14045 | 645 |
lemma eval_conf: "\<lbrakk>G \<turnstile> s -e\<succ>v-> s'; wf_java_prog G; s::\<preceq>E; |
13673 | 646 |
E\<turnstile>e::T; gx s' = None; prg E = G \<rbrakk> |
647 |
\<Longrightarrow> G,gh s'\<turnstile>v::\<preceq>T" |
|
648 |
apply (simp add: gh_def) |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
649 |
apply (rule_tac x3="fst s" and s3="snd s"and x'3="fst s'" |
14143 | 650 |
in eval_type_sound [THEN conjunct2 [THEN conjunct1 [THEN mp]], simplified]) |
651 |
apply assumption+ |
|
13673 | 652 |
apply (simp (no_asm_use) add: surjective_pairing [THEN sym]) |
14045 | 653 |
apply (simp only: surjective_pairing [THEN sym]) |
654 |
apply (auto simp add: gs_def gx_def) |
|
13673 | 655 |
done |
656 |
||
657 |
lemma evals_preserves_conf: |
|
658 |
"\<lbrakk> G\<turnstile> s -es[\<succ>]vs-> s'; G,gh s \<turnstile> t ::\<preceq> T; E \<turnstile>es[::]Ts; |
|
14045 | 659 |
wf_java_prog G; s::\<preceq>E; |
13673 | 660 |
prg E = G \<rbrakk> \<Longrightarrow> G,gh s' \<turnstile> t ::\<preceq> T" |
661 |
apply (subgoal_tac "gh s\<le>| gh s'") |
|
662 |
apply (frule conf_hext, assumption, assumption) |
|
663 |
apply (frule eval_evals_exec_type_sound [THEN conjunct2 [THEN conjunct1 [THEN mp]]]) |
|
664 |
apply (subgoal_tac "G \<turnstile> (gx s, (gh s, gl s)) -es[\<succ>]vs-> (gx s', (gh s', gl s'))") |
|
665 |
apply assumption |
|
666 |
apply (simp add: gx_def gh_def gl_def surjective_pairing [THEN sym]) |
|
667 |
apply (case_tac E) |
|
14045 | 668 |
apply (simp add: gx_def gs_def gh_def gl_def surjective_pairing [THEN sym]) |
13673 | 669 |
done |
670 |
||
671 |
lemma eval_of_class: "\<lbrakk> G \<turnstile> s -e\<succ>a'-> s'; E \<turnstile> e :: Class C; |
|
14045 | 672 |
wf_java_prog G; s::\<preceq>E; gx s'=None; a' \<noteq> Null; G=prg E\<rbrakk> |
13673 | 673 |
\<Longrightarrow> (\<exists> lc. a' = Addr lc)" |
674 |
apply (case_tac s, case_tac s', simp) |
|
14045 | 675 |
apply (frule eval_type_sound, (simp add: gs_def)+) |
13673 | 676 |
apply (case_tac a') |
677 |
apply (auto simp: conf_def) |
|
678 |
done |
|
679 |
||
680 |
||
681 |
lemma dynT_subcls: |
|
682 |
"\<lbrakk> a' \<noteq> Null; G,h\<turnstile>a'::\<preceq> Class C; dynT = fst (the (h (the_Addr a'))); |
|
14045 | 683 |
is_class G dynT; ws_prog G \<rbrakk> \<Longrightarrow> G\<turnstile>dynT \<preceq>C C" |
13673 | 684 |
apply (case_tac "C = Object") |
685 |
apply (simp, rule subcls_C_Object, assumption+) |
|
14045 | 686 |
apply simp |
13673 | 687 |
apply (frule non_np_objD, auto) |
688 |
done |
|
689 |
||
690 |
||
691 |
lemma method_defined: "\<lbrakk> |
|
692 |
m = the (method (G, dynT) (mn, pTs)); |
|
693 |
dynT = fst (the (h a)); is_class G dynT; wf_java_prog G; |
|
694 |
a' \<noteq> Null; G,h\<turnstile>a'::\<preceq> Class C; a = the_Addr a'; |
|
695 |
\<exists>pTsa md rT. max_spec G C (mn, pTsa) = {((md, rT), pTs)} \<rbrakk> |
|
696 |
\<Longrightarrow> (method (G, dynT) (mn, pTs)) = Some m" |
|
697 |
apply (erule exE)+ |
|
698 |
apply (drule singleton_in_set, drule max_spec2appl_meths) |
|
699 |
apply (simp add: appl_methds_def) |
|
700 |
apply ((erule exE)+, (erule conjE)+, (erule exE)+) |
|
701 |
apply (drule widen_methd) |
|
702 |
apply assumption |
|
14045 | 703 |
apply (rule dynT_subcls) apply assumption+ apply simp apply simp |
13673 | 704 |
apply (erule exE)+ apply simp |
705 |
done |
|
706 |
||
707 |
||
708 |
||
709 |
(**********************************************************************) |
|
710 |
||
711 |
||
712 |
(* 1. any difference between locvars_xstate \<dots> and L ??? *) |
|
713 |
(* 2. possibly skip env_of_jmb ??? *) |
|
714 |
theorem compiler_correctness: |
|
715 |
"wf_java_prog G \<Longrightarrow> |
|
22271 | 716 |
(G \<turnstile> xs -ex\<succ>val-> xs' \<longrightarrow> |
13673 | 717 |
gx xs = None \<longrightarrow> gx xs' = None \<longrightarrow> |
718 |
(\<forall> os CL S. |
|
719 |
(class_sig_defined G CL S) \<longrightarrow> |
|
720 |
(wtpd_expr (env_of_jmb G CL S) ex) \<longrightarrow> |
|
14045 | 721 |
(xs ::\<preceq> (env_of_jmb G CL S)) \<longrightarrow> |
13673 | 722 |
( {TranslComp.comp G, CL, S} \<turnstile> |
723 |
{gh xs, os, (locvars_xstate G CL S xs)} |
|
724 |
>- (compExpr (gmb G CL S) ex) \<rightarrow> |
|
725 |
{gh xs', val#os, locvars_xstate G CL S xs'}))) \<and> |
|
726 |
||
22271 | 727 |
(G \<turnstile> xs -exs[\<succ>]vals-> xs' \<longrightarrow> |
13673 | 728 |
gx xs = None \<longrightarrow> gx xs' = None \<longrightarrow> |
729 |
(\<forall> os CL S. |
|
730 |
(class_sig_defined G CL S) \<longrightarrow> |
|
731 |
(wtpd_exprs (env_of_jmb G CL S) exs) \<longrightarrow> |
|
14045 | 732 |
(xs::\<preceq>(env_of_jmb G CL S)) \<longrightarrow> |
13673 | 733 |
( {TranslComp.comp G, CL, S} \<turnstile> |
734 |
{gh xs, os, (locvars_xstate G CL S xs)} |
|
735 |
>- (compExprs (gmb G CL S) exs) \<rightarrow> |
|
736 |
{gh xs', (rev vals)@os, (locvars_xstate G CL S xs')}))) \<and> |
|
737 |
||
22271 | 738 |
(G \<turnstile> xs -st-> xs' \<longrightarrow> |
13673 | 739 |
gx xs = None \<longrightarrow> gx xs' = None \<longrightarrow> |
740 |
(\<forall> os CL S. |
|
741 |
(class_sig_defined G CL S) \<longrightarrow> |
|
742 |
(wtpd_stmt (env_of_jmb G CL S) st) \<longrightarrow> |
|
14045 | 743 |
(xs::\<preceq>(env_of_jmb G CL S)) \<longrightarrow> |
13673 | 744 |
( {TranslComp.comp G, CL, S} \<turnstile> |
745 |
{gh xs, os, (locvars_xstate G CL S xs)} |
|
746 |
>- (compStmt (gmb G CL S) st) \<rightarrow> |
|
747 |
{gh xs', os, (locvars_xstate G CL S xs')})))" |
|
748 |
apply (rule Eval.eval_evals_exec.induct) |
|
749 |
||
750 |
(* case XcptE *) |
|
751 |
apply simp |
|
752 |
||
753 |
(* case NewC *) |
|
14045 | 754 |
apply clarify |
755 |
apply (frule wf_prog_ws_prog [THEN wf_subcls1]) (* establish wf ((subcls1 G)^-1) *) |
|
13673 | 756 |
apply (simp add: c_hupd_hp_invariant) |
757 |
apply (rule progression_one_step) |
|
758 |
apply (rotate_tac 1, drule sym) (* reverse equation (a, None) = new_Addr (fst s) *) |
|
759 |
apply (simp add: locvars_xstate_def locvars_locals_def comp_fields) |
|
760 |
||
761 |
||
762 |
(* case Cast *) |
|
763 |
apply (intro allI impI) |
|
764 |
apply simp |
|
765 |
apply (frule raise_if_NoneD) |
|
766 |
apply (frule wtpd_expr_cast) |
|
767 |
apply simp |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
768 |
apply (rule_tac ?instrs0.0 = "(compExpr (gmb G CL S) e)" in progression_transitive, simp) |
13673 | 769 |
apply blast |
770 |
apply (rule progression_one_step) |
|
771 |
apply (simp add: raise_system_xcpt_def gh_def comp_cast_ok) |
|
772 |
||
773 |
||
774 |
(* case Lit *) |
|
775 |
apply simp |
|
776 |
apply (intro strip) |
|
777 |
apply (rule progression_one_step) |
|
778 |
apply simp |
|
779 |
||
780 |
||
781 |
(* case BinOp *) |
|
782 |
apply (intro allI impI) |
|
783 |
apply (frule_tac xs=s1 in eval_xcpt, assumption) (* establish (gx s1 = None) *) |
|
784 |
apply (frule wtpd_expr_binop) |
|
14045 | 785 |
(* establish (s1::\<preceq> \<dots>) *) |
13673 | 786 |
apply (frule_tac e=e1 in state_ok_eval) apply (simp (no_asm_simp)) apply simp apply (simp (no_asm_use) only: env_of_jmb_fst) |
787 |
||
788 |
||
789 |
apply (simp (no_asm_use) only: compExpr_compExprs.simps) |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
790 |
apply (rule_tac ?instrs0.0 = "compExpr (gmb G CL S) e1" in progression_transitive, simp) apply blast |
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
791 |
apply (rule_tac ?instrs0.0 = "compExpr (gmb G CL S) e2" in progression_transitive, simp) apply blast |
13673 | 792 |
apply (case_tac bop) |
793 |
(*subcase bop = Eq *) apply simp apply (rule progression_Eq) |
|
794 |
(*subcase bop = Add *) apply simp apply (rule progression_one_step) apply simp |
|
795 |
||
796 |
||
797 |
(* case LAcc *) |
|
798 |
apply simp |
|
799 |
apply (intro strip) |
|
800 |
apply (rule progression_one_step) |
|
801 |
apply (simp add: locvars_xstate_def locvars_locals_def) |
|
802 |
apply (frule wtpd_expr_lacc) |
|
803 |
apply assumption |
|
804 |
apply (simp add: gl_def) |
|
805 |
apply (erule select_at_index) |
|
806 |
||
807 |
||
808 |
(* case LAss *) |
|
809 |
apply (intro allI impI) |
|
810 |
apply (frule wtpd_expr_lass, erule conjE, erule conjE) |
|
46226 | 811 |
apply simp |
13673 | 812 |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
813 |
apply (rule_tac ?instrs0.0 = "(compExpr (gmb G CL S) e)" in progression_transitive, rule HOL.refl) |
13673 | 814 |
apply blast |
815 |
||
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
816 |
apply (rule_tac ?instrs0.0 = "[Dup]" in progression_transitive, simp) |
13673 | 817 |
apply (rule progression_one_step) |
818 |
apply (simp add: gh_def) |
|
819 |
apply (rule conjI, simp)+ apply simp |
|
820 |
apply (rule progression_one_step) |
|
821 |
apply (simp add: gh_def) |
|
822 |
(* the following falls out of the general scheme *) |
|
823 |
apply (frule wtpd_expr_lacc) apply assumption |
|
824 |
apply (rule update_at_index) |
|
825 |
apply (rule distinct_method_if_class_sig_defined) apply assumption |
|
826 |
apply assumption apply simp apply assumption |
|
827 |
||
828 |
||
829 |
(* case FAcc *) |
|
830 |
apply (intro allI impI) |
|
831 |
(* establish x1 = None \<and> a' \<noteq> Null *) |
|
832 |
apply (simp (no_asm_use) only: gx_conv, frule np_NoneD) |
|
833 |
apply (frule wtpd_expr_facc) |
|
834 |
||
835 |
apply (simp (no_asm_use) only: compExpr_compExprs.simps) |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
836 |
apply (rule_tac ?instrs0.0 = "(compExpr (gmb G CL S) e)" in progression_transitive, rule HOL.refl) |
13673 | 837 |
apply blast |
838 |
apply (rule progression_one_step) |
|
839 |
apply (simp add: gh_def) |
|
840 |
apply (case_tac "(the (fst s1 (the_Addr a')))") |
|
841 |
apply (simp add: raise_system_xcpt_def) |
|
842 |
||
843 |
||
844 |
(* case FAss *) |
|
845 |
apply (intro allI impI) |
|
846 |
apply (frule wtpd_expr_fass) apply (erule conjE) apply (frule wtpd_expr_facc) |
|
847 |
apply (simp only: c_hupd_xcpt_invariant) (* establish x2 = None *) |
|
848 |
(* establish x1 = None and a' \<noteq> Null *) |
|
849 |
apply (frule_tac xs="(np a' x1, s1)" in eval_xcpt) |
|
850 |
apply (simp only: gx_conv, simp only: gx_conv, frule np_NoneD, erule conjE) |
|
851 |
||
852 |
||
14045 | 853 |
(* establish ((Norm s1)::\<preceq> \<dots>) *) |
854 |
apply (frule_tac e=e1 in state_ok_eval) apply (simp (no_asm_simp) only: env_of_jmb_fst) |
|
855 |
apply assumption apply (simp (no_asm_use) only: env_of_jmb_fst) |
|
13673 | 856 |
|
857 |
apply (simp only: compExpr_compExprs.simps) |
|
858 |
||
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
859 |
apply (rule_tac ?instrs0.0 = "(compExpr (gmb G CL S) e1)" in progression_transitive, rule HOL.refl) |
13673 | 860 |
apply fast (* blast does not seem to work - why? *) |
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
861 |
apply (rule_tac ?instrs0.0 = "(compExpr (gmb G CL S) e2)" in progression_transitive, rule HOL.refl) |
13673 | 862 |
apply fast |
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
863 |
apply (rule_tac ?instrs0.0 = "[Dup_x1]" and ?instrs1.0 = "[Putfield fn T]" in progression_transitive, simp) |
13673 | 864 |
|
865 |
(* Dup_x1 *) |
|
866 |
apply (rule progression_one_step) |
|
867 |
apply (simp add: gh_def) |
|
868 |
apply (rule conjI, simp)+ apply simp |
|
869 |
||
870 |
||
871 |
(* Putfield \<longrightarrow> still looks nasty*) |
|
872 |
apply (rule progression_one_step) |
|
873 |
apply simp |
|
874 |
apply (case_tac "(the (fst s2 (the_Addr a')))") |
|
875 |
apply (simp add: c_hupd_hp_invariant) |
|
876 |
apply (case_tac s2) |
|
877 |
apply (simp add: c_hupd_conv raise_system_xcpt_def) |
|
878 |
apply (rule locvars_xstate_par_dep, rule HOL.refl) |
|
879 |
||
880 |
defer (* method call *) |
|
881 |
||
882 |
(* case XcptEs *) |
|
883 |
apply simp |
|
884 |
||
885 |
(* case Nil *) |
|
46226 | 886 |
apply simp |
13673 | 887 |
apply (intro strip) |
888 |
apply (rule progression_refl) |
|
889 |
||
890 |
(* case Cons *) |
|
891 |
apply (intro allI impI) |
|
892 |
apply (frule_tac xs=s1 in evals_xcpt, simp only: gx_conv) (* establish gx s1 = None *) |
|
893 |
apply (frule wtpd_exprs_cons) |
|
14045 | 894 |
(* establish ((Norm s0)::\<preceq> \<dots>) *) |
13673 | 895 |
apply (frule_tac e=e in state_ok_eval) apply (simp (no_asm_simp) only: env_of_jmb_fst) apply simp apply (simp (no_asm_use) only: env_of_jmb_fst) |
896 |
||
897 |
apply simp |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
898 |
apply (rule_tac ?instrs0.0 = "(compExpr (gmb G CL S) e)" in progression_transitive, rule HOL.refl) |
13673 | 899 |
apply fast |
900 |
apply fast |
|
901 |
||
902 |
||
903 |
(* case Statement: exception *) |
|
904 |
apply simp |
|
905 |
||
906 |
(* case Skip *) |
|
907 |
apply (intro allI impI) |
|
908 |
apply simp |
|
909 |
apply (rule progression_refl) |
|
910 |
||
911 |
(* case Expr *) |
|
912 |
apply (intro allI impI) |
|
913 |
apply (frule wtpd_stmt_expr) |
|
914 |
apply simp |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
915 |
apply (rule_tac ?instrs0.0 = "(compExpr (gmb G CL S) e)" in progression_transitive, rule HOL.refl) |
13673 | 916 |
apply fast |
917 |
apply (rule progression_one_step) |
|
918 |
apply simp |
|
919 |
||
920 |
(* case Comp *) |
|
921 |
apply (intro allI impI) |
|
922 |
apply (frule_tac xs=s1 in exec_xcpt, assumption) (* establish (gx s1 = None) *) |
|
923 |
apply (frule wtpd_stmt_comp) |
|
924 |
||
14045 | 925 |
(* establish (s1::\<preceq> \<dots>) *) |
13673 | 926 |
apply (frule_tac st=c1 in state_ok_exec) apply (simp (no_asm_simp) only: env_of_jmb_fst) apply simp apply (simp (no_asm_use) only: env_of_jmb_fst) |
927 |
||
928 |
apply simp |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
929 |
apply (rule_tac ?instrs0.0 = "(compStmt (gmb G CL S) c1)" in progression_transitive, rule HOL.refl) |
13673 | 930 |
apply fast |
931 |
apply fast |
|
932 |
||
933 |
||
934 |
(* case Cond *) |
|
935 |
apply (intro allI impI) |
|
936 |
apply (frule_tac xs=s1 in exec_xcpt, assumption) (* establish (gx s1 = None) *) |
|
937 |
apply (frule wtpd_stmt_cond, (erule conjE)+) |
|
14045 | 938 |
(* establish (s1::\<preceq> \<dots>) *) |
13673 | 939 |
apply (frule_tac e=e in state_ok_eval) |
940 |
apply (simp (no_asm_simp) only: env_of_jmb_fst) |
|
941 |
apply assumption |
|
942 |
apply (simp (no_asm_use) only: env_of_jmb_fst) |
|
943 |
(* establish G,gh s1\<turnstile>v::\<preceq>PrimT Boolean *) |
|
944 |
apply (frule eval_conf, assumption+, rule env_of_jmb_fst) |
|
945 |
apply (frule conf_bool) (* establish \<exists>b. v = Bool b *) |
|
946 |
apply (erule exE) |
|
947 |
||
948 |
apply simp |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
949 |
apply (rule_tac ?instrs0.0 = "[LitPush (Bool False)]" in progression_transitive, simp (no_asm_simp)) |
13673 | 950 |
apply (rule progression_one_step, simp) |
951 |
apply (rule conjI, rule HOL.refl)+ apply (rule HOL.refl) |
|
952 |
||
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
953 |
apply (rule_tac ?instrs0.0 = "compExpr (gmb G CL S) e" in progression_transitive, rule HOL.refl) |
13673 | 954 |
apply fast |
955 |
||
956 |
apply (case_tac b) |
|
957 |
(* case b= True *) |
|
958 |
apply simp |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
959 |
apply (rule_tac ?instrs0.0 = "[Ifcmpeq (2 + int (length (compStmt (gmb G CL S) c1)))]" in progression_transitive, simp) |
13673 | 960 |
apply (rule progression_one_step) apply simp |
961 |
apply (rule conjI, rule HOL.refl)+ apply (rule HOL.refl) |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
962 |
apply (rule_tac ?instrs0.0 = "(compStmt (gmb G CL S) c1)" in progression_transitive, simp) |
13673 | 963 |
apply fast |
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
964 |
apply (rule_tac ?instrs1.0 = "[]" in jump_fwd_progression) |
13673 | 965 |
apply (simp, rule conjI, (rule HOL.refl)+) |
20432
07ec57376051
lin_arith_prover: splitting reverted because of performance loss
webertj
parents:
20272
diff
changeset
|
966 |
apply simp apply (rule conjI, simp) apply (simp add: nat_add_distrib) |
13673 | 967 |
apply (rule progression_refl) |
968 |
||
969 |
(* case b= False *) |
|
970 |
apply simp |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
971 |
apply (rule_tac ?instrs1.0 = "compStmt (gmb G CL S) c2" in jump_fwd_progression) |
13673 | 972 |
apply (simp, rule conjI, (rule HOL.refl)+) |
20432
07ec57376051
lin_arith_prover: splitting reverted because of performance loss
webertj
parents:
20272
diff
changeset
|
973 |
apply (simp, rule conjI, rule HOL.refl, simp add: nat_add_distrib) |
13673 | 974 |
apply fast |
975 |
||
976 |
(* case exit Loop *) |
|
977 |
apply (intro allI impI) |
|
978 |
apply (frule wtpd_stmt_loop, (erule conjE)+) |
|
979 |
||
980 |
(* establish G,gh s1\<turnstile>v::\<preceq>PrimT Boolean *) |
|
981 |
apply (frule eval_conf, assumption+, rule env_of_jmb_fst) |
|
982 |
apply (frule conf_bool) (* establish \<exists>b. v = Bool b *) |
|
983 |
apply (erule exE) |
|
984 |
apply (case_tac b) |
|
985 |
||
986 |
(* case b= True \<longrightarrow> contradiction *) |
|
987 |
apply simp |
|
988 |
||
989 |
(* case b= False *) |
|
990 |
apply simp |
|
991 |
||
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
992 |
apply (rule_tac ?instrs0.0 = "[LitPush (Bool False)]" in progression_transitive, simp (no_asm_simp)) |
13673 | 993 |
apply (rule progression_one_step) |
994 |
apply simp |
|
995 |
apply (rule conjI, rule HOL.refl)+ apply (rule HOL.refl) |
|
996 |
||
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
997 |
apply (rule_tac ?instrs0.0 = "compExpr (gmb G CL S) e" in progression_transitive, rule HOL.refl) |
13673 | 998 |
apply fast |
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
999 |
apply (rule_tac ?instrs1.0 = "[]" in jump_fwd_progression) |
13673 | 1000 |
apply (simp, rule conjI, rule HOL.refl, rule HOL.refl) |
20432
07ec57376051
lin_arith_prover: splitting reverted because of performance loss
webertj
parents:
20272
diff
changeset
|
1001 |
apply (simp, rule conjI, rule HOL.refl, simp add: nat_add_distrib) |
13673 | 1002 |
apply (rule progression_refl) |
1003 |
||
1004 |
||
1005 |
(* case continue Loop *) |
|
1006 |
apply (intro allI impI) |
|
1007 |
apply (frule_tac xs=s2 in exec_xcpt, assumption) (* establish (gx s2 = None) *) |
|
1008 |
apply (frule_tac xs=s1 in exec_xcpt, assumption) (* establish (gx s1 = None) *) |
|
1009 |
apply (frule wtpd_stmt_loop, (erule conjE)+) |
|
1010 |
||
14045 | 1011 |
(* establish (s1::\<preceq> \<dots>) *) |
13673 | 1012 |
apply (frule_tac e=e in state_ok_eval) apply (simp (no_asm_simp) only: env_of_jmb_fst) apply simp apply (simp (no_asm_use) only: env_of_jmb_fst) |
14045 | 1013 |
(* establish (s2::\<preceq> \<dots>) *) |
13673 | 1014 |
apply (frule_tac xs=s1 and st=c in state_ok_exec) |
1015 |
apply (simp (no_asm_simp) only: env_of_jmb_fst) apply assumption apply (simp (no_asm_use) only: env_of_jmb_fst) |
|
1016 |
||
1017 |
(* establish G,gh s1\<turnstile>v::\<preceq>PrimT Boolean *) |
|
1018 |
apply (frule eval_conf, assumption+, rule env_of_jmb_fst) |
|
1019 |
apply (frule conf_bool) (* establish \<exists>b. v = Bool b *) |
|
1020 |
apply (erule exE) |
|
1021 |
||
1022 |
apply simp |
|
1023 |
apply (rule jump_bwd_progression) |
|
1024 |
apply simp |
|
1025 |
apply (rule conjI, (rule HOL.refl)+) |
|
1026 |
||
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
1027 |
apply (rule_tac ?instrs0.0 = "[LitPush (Bool False)]" in progression_transitive, simp (no_asm_simp)) |
13673 | 1028 |
apply (rule progression_one_step) |
1029 |
apply simp |
|
1030 |
apply (rule conjI, simp)+ apply simp |
|
1031 |
||
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
1032 |
apply (rule_tac ?instrs0.0 = "compExpr (gmb G CL S) e" in progression_transitive, rule HOL.refl) |
13673 | 1033 |
apply fast |
1034 |
||
1035 |
apply (case_tac b) |
|
1036 |
(* case b= True *) |
|
1037 |
apply simp |
|
1038 |
||
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
1039 |
apply (rule_tac ?instrs0.0 = "[Ifcmpeq (2 + int (length (compStmt (gmb G CL S) c)))]" in progression_transitive, simp) |
13673 | 1040 |
apply (rule progression_one_step) apply simp |
1041 |
apply (rule conjI, rule HOL.refl)+ apply (rule HOL.refl) |
|
1042 |
apply fast |
|
1043 |
||
1044 |
(* case b= False \<longrightarrow> contradiction*) |
|
1045 |
apply simp |
|
1046 |
||
1047 |
apply (rule jump_bwd_one_step) |
|
1048 |
apply simp |
|
1049 |
apply blast |
|
1050 |
||
1051 |
(*****) |
|
14045 | 1052 |
(* case method call *) |
13673 | 1053 |
|
1054 |
apply (intro allI impI) |
|
1055 |
||
1056 |
apply (frule_tac xs=s3 in eval_xcpt, simp only: gx_conv) (* establish gx s3 = None *) |
|
1057 |
apply (frule exec_xcpt, assumption, simp (no_asm_use) only: gx_conv, frule np_NoneD) (* establish x = None \<and> a' \<noteq> Null *) |
|
1058 |
apply (frule evals_xcpt, simp only: gx_conv) (* establish gx s1 = None *) |
|
1059 |
||
1060 |
apply (frule wtpd_expr_call, (erule conjE)+) |
|
1061 |
||
1062 |
||
1063 |
(* assumptions about state_ok and is_class *) |
|
1064 |
||
14045 | 1065 |
(* establish s1::\<preceq> (env_of_jmb G CL S) *) |
13673 | 1066 |
apply (frule_tac xs="Norm s0" and e=e in state_ok_eval) |
1067 |
apply (simp (no_asm_simp) only: env_of_jmb_fst, assumption, simp (no_asm_use) only: env_of_jmb_fst) |
|
1068 |
||
14045 | 1069 |
(* establish (x, h, l)::\<preceq>(env_of_jmb G CL S) *) |
13673 | 1070 |
apply (frule_tac xs=s1 and xs'="(x, h, l)" in state_ok_evals) |
1071 |
apply (simp (no_asm_simp) only: env_of_jmb_fst, assumption, simp only: env_of_jmb_fst) |
|
1072 |
||
1073 |
(* establish \<exists> lc. a' = Addr lc *) |
|
1074 |
apply (frule (5) eval_of_class, rule env_of_jmb_fst [THEN sym]) |
|
1075 |
apply (subgoal_tac "G,h \<turnstile> a' ::\<preceq> Class C") |
|
1076 |
apply (subgoal_tac "is_class G dynT") |
|
1077 |
||
1078 |
(* establish method (G, dynT) (mn, pTs) = Some(md, rT, pns, lvars, blk, res) *) |
|
1079 |
apply (drule method_defined, assumption+) |
|
1080 |
apply (simp only: env_of_jmb_fst) |
|
1081 |
apply ((erule exE)+, erule conjE, (rule exI)+, assumption) |
|
1082 |
||
1083 |
apply (subgoal_tac "is_class G md") |
|
1084 |
apply (subgoal_tac "G\<turnstile>Class dynT \<preceq> Class md") |
|
1085 |
apply (subgoal_tac " method (G, md) (mn, pTs) = Some (md, rT, pns, lvars, blk, res)") |
|
1086 |
apply (subgoal_tac "list_all2 (conf G h) pvs pTs") |
|
1087 |
||
14045 | 1088 |
(* establish (np a' x, h, init_vars lvars(pns[\<mapsto>]pvs)(This\<mapsto>a'))::\<preceq>(env_of_jmb G md (mn, pTs)) *) |
13673 | 1089 |
apply (subgoal_tac "G,h \<turnstile> a' ::\<preceq> Class dynT") |
1090 |
apply (frule (2) conf_widen) |
|
1091 |
apply (frule state_ok_init, assumption+) |
|
1092 |
||
1093 |
apply (subgoal_tac "class_sig_defined G md (mn, pTs)") |
|
1094 |
apply (frule wtpd_blk, assumption, assumption) |
|
1095 |
apply (frule wtpd_res, assumption, assumption) |
|
14045 | 1096 |
apply (subgoal_tac "s3::\<preceq>(env_of_jmb G md (mn, pTs))") |
13673 | 1097 |
|
14045 | 1098 |
apply (subgoal_tac "method (TranslComp.comp G, md) (mn, pTs) = |
1099 |
Some (md, rT, snd (snd (compMethod G md ((mn, pTs), rT, pns, lvars, blk, res))))") |
|
1100 |
prefer 2 apply (simp add: wf_prog_ws_prog [THEN comp_method]) |
|
1101 |
apply (subgoal_tac "method (TranslComp.comp G, dynT) (mn, pTs) = |
|
1102 |
Some (md, rT, snd (snd (compMethod G md ((mn, pTs), rT, pns, lvars, blk, res))))") |
|
1103 |
prefer 2 apply (simp add: wf_prog_ws_prog [THEN comp_method]) |
|
13673 | 1104 |
apply (simp only: fst_conv snd_conv) |
1105 |
||
1106 |
(* establish length pns = length pTs *) |
|
1107 |
apply (frule method_preserves_length, assumption, assumption) |
|
1108 |
(* establish length pvs = length ps *) |
|
1109 |
apply (frule evals_preserves_length [THEN sym]) |
|
1110 |
||
1111 |
(** start evaluating subexpressions **) |
|
1112 |
apply (simp (no_asm_use) only: compExpr_compExprs.simps) |
|
1113 |
||
1114 |
(* evaluate e *) |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
1115 |
apply (rule_tac ?instrs0.0 = "(compExpr (gmb G CL S) e)" in progression_transitive, rule HOL.refl) |
13673 | 1116 |
apply fast |
1117 |
||
1118 |
(* evaluate parameters *) |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
1119 |
apply (rule_tac ?instrs0.0 = "compExprs (gmb G CL S) ps" in progression_transitive, rule HOL.refl) |
13673 | 1120 |
apply fast |
1121 |
||
1122 |
(* invokation *) |
|
1123 |
apply (rule progression_call) |
|
1124 |
apply (intro allI impI conjI) |
|
1125 |
(* execute Invoke statement *) |
|
1126 |
apply (simp (no_asm_use) only: exec_instr.simps) |
|
1127 |
apply (erule thin_rl, erule thin_rl, erule thin_rl) |
|
1128 |
apply (simp add: compMethod_def raise_system_xcpt_def) |
|
1129 |
apply (rule conjI, simp)+ apply (rule HOL.refl) |
|
1130 |
||
1131 |
(* get instructions of invoked method *) |
|
1132 |
apply (simp (no_asm_simp) add: gis_def gmb_def compMethod_def) |
|
1133 |
||
1134 |
(* var. initialization *) |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
1135 |
apply (rule_tac ?instrs0.0 = "(compInitLvars (pns, lvars, blk, res) lvars)" in progression_transitive, rule HOL.refl) |
13673 | 1136 |
apply (rule_tac C=md in progression_lvar_init, assumption, assumption, assumption) |
1137 |
apply (simp (no_asm_simp)) (* length pns = length pvs *) |
|
28524 | 1138 |
apply (simp (no_asm_simp)) (* length lvars = length (replicate (length lvars) undefined) *) |
13673 | 1139 |
|
1140 |
||
1141 |
(* body statement *) |
|
14174
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
ballarin
parents:
14143
diff
changeset
|
1142 |
apply (rule_tac ?instrs0.0 = "compStmt (pns, lvars, blk, res) blk" in progression_transitive, rule HOL.refl) |
13673 | 1143 |
apply (subgoal_tac "(pns, lvars, blk, res) = gmb G md (mn, pTs)") |
1144 |
apply (simp (no_asm_simp)) |
|
15866 | 1145 |
apply (simp only: gh_conv) |
1146 |
apply (drule mp [OF _ TrueI])+ |
|
1147 |
apply (erule allE, erule allE, erule allE, erule impE, assumption)+ |
|
1148 |
apply ((erule impE, assumption)+, assumption) |
|
15860 | 1149 |
|
13673 | 1150 |
apply (simp (no_asm_use)) |
1151 |
apply (simp (no_asm_simp) add: gmb_def) |
|
1152 |
||
1153 |
(* return expression *) |
|
1154 |
apply (subgoal_tac "(pns, lvars, blk, res) = gmb G md (mn, pTs)") |
|
1155 |
apply (simp (no_asm_simp)) |
|
1156 |
apply (simp only: gh_conv) |
|
1157 |
apply ((drule mp, rule TrueI)+, (drule spec)+, (drule mp, assumption)+, assumption) |
|
1158 |
apply (simp (no_asm_use)) |
|
1159 |
apply (simp (no_asm_simp) add: gmb_def) |
|
1160 |
||
1161 |
(* execute return statement *) |
|
1162 |
apply (simp (no_asm_use) add: gh_def locvars_xstate_def gl_def del: drop_append) |
|
1163 |
apply (subgoal_tac "rev pvs @ a' # os = (rev (a' # pvs)) @ os") |
|
1164 |
apply (simp only: drop_append) |
|
1165 |
apply (simp (no_asm_simp)) |
|
1166 |
apply (simp (no_asm_simp)) |
|
1167 |
||
14045 | 1168 |
(* show s3::\<preceq>\<dots> *) |
13673 | 1169 |
apply (rule_tac xs = "(np a' x, h, init_vars lvars(pns[\<mapsto>]pvs)(This\<mapsto>a'))" and st=blk in state_ok_exec) |
1170 |
apply assumption apply (simp (no_asm_simp) only: env_of_jmb_fst) |
|
1171 |
apply assumption apply (simp (no_asm_use) only: env_of_jmb_fst) |
|
1172 |
||
1173 |
(* show class_sig_defined G md (mn, pTs) *) |
|
1174 |
apply (simp (no_asm_simp) add: class_sig_defined_def) |
|
1175 |
||
1176 |
(* show G,h \<turnstile> a' ::\<preceq> Class dynT *) |
|
1177 |
apply (frule non_npD) apply assumption |
|
1178 |
apply (erule exE)+ apply simp |
|
1179 |
apply (rule conf_obj_AddrI) apply simp |
|
1180 |
apply (rule conjI, (rule HOL.refl)+) |
|
1181 |
apply (rule widen_Class_Class [THEN iffD1], rule widen.refl) |
|
1182 |
||
1183 |
||
1184 |
(* show list_all2 (conf G h) pvs pTs *) |
|
1185 |
apply (erule exE)+ apply (erule conjE)+ |
|
1186 |
apply (rule_tac Ts="pTsa" in conf_list_gext_widen) apply assumption |
|
22271 | 1187 |
apply (subgoal_tac "G \<turnstile> (gx s1, gs s1) -ps[\<succ>]pvs-> (x, h, l)") |
13673 | 1188 |
apply (frule_tac E="env_of_jmb G CL S" in evals_type_sound) |
14143 | 1189 |
apply assumption+ |
13673 | 1190 |
apply (simp only: env_of_jmb_fst) |
1191 |
apply (simp add: conforms_def xconf_def gs_def) |
|
1192 |
apply simp |
|
1193 |
apply (simp (no_asm_use) only: gx_def gs_def surjective_pairing [THEN sym]) |
|
1194 |
apply (simp (no_asm_use) only: ty_exprs_list_all2) apply simp |
|
14143 | 1195 |
apply simp |
13673 | 1196 |
apply (simp (no_asm_use) only: gx_def gs_def surjective_pairing [THEN sym]) |
1197 |
(* list_all2 (\<lambda>T T'. G \<turnstile> T \<preceq> T') pTsa pTs *) |
|
1198 |
apply (rule max_spec_widen, simp only: env_of_jmb_fst) |
|
1199 |
||
1200 |
||
1201 |
(* show method (G, md) (mn, pTs) = Some (md, rT, pns, lvars, blk, res) *) |
|
14045 | 1202 |
apply (frule wf_prog_ws_prog [THEN method_in_md [THEN conjunct2]], assumption+) |
13673 | 1203 |
|
1204 |
(* show G\<turnstile>Class dynT \<preceq> Class md *) |
|
1205 |
apply (simp (no_asm_use) only: widen_Class_Class) |
|
1206 |
apply (rule method_wf_mdecl [THEN conjunct1], assumption+) |
|
1207 |
||
1208 |
(* is_class G md *) |
|
14045 | 1209 |
apply (rule wf_prog_ws_prog [THEN method_in_md [THEN conjunct1]], assumption+) |
13673 | 1210 |
|
1211 |
(* show is_class G dynT *) |
|
1212 |
apply (frule non_npD) apply assumption |
|
1213 |
apply (erule exE)+ apply (erule conjE)+ |
|
1214 |
apply simp |
|
1215 |
apply (rule subcls_is_class2) apply assumption |
|
1216 |
apply (frule class_expr_is_class) apply (simp only: env_of_jmb_fst) |
|
14045 | 1217 |
apply (rule wf_prog_ws_prog, assumption) |
13673 | 1218 |
apply (simp only: env_of_jmb_fst) |
1219 |
||
1220 |
(* show G,h \<turnstile> a' ::\<preceq> Class C *) |
|
1221 |
apply (simp only: wtpd_exprs_def, erule exE) |
|
1222 |
apply (frule evals_preserves_conf) |
|
1223 |
apply (rule eval_conf, assumption+) |
|
1224 |
apply (rule env_of_jmb_fst, assumption+) |
|
1225 |
apply (rule env_of_jmb_fst) |
|
1226 |
apply (simp only: gh_conv) |
|
1227 |
done |
|
1228 |
||
1229 |
||
1230 |
theorem compiler_correctness_eval: " |
|
1231 |
\<lbrakk> G \<turnstile> (None,hp,loc) -ex \<succ> val-> (None,hp',loc'); |
|
1232 |
wf_java_prog G; |
|
1233 |
class_sig_defined G C S; |
|
1234 |
wtpd_expr (env_of_jmb G C S) ex; |
|
1235 |
(None,hp,loc) ::\<preceq> (env_of_jmb G C S) \<rbrakk> \<Longrightarrow> |
|
1236 |
{(TranslComp.comp G), C, S} \<turnstile> |
|
1237 |
{hp, os, (locvars_locals G C S loc)} |
|
1238 |
>- (compExpr (gmb G C S) ex) \<rightarrow> |
|
1239 |
{hp', val#os, (locvars_locals G C S loc')}" |
|
1240 |
apply (frule compiler_correctness [THEN conjunct1]) |
|
14045 | 1241 |
apply (auto simp: gh_def gx_def gs_def gl_def locvars_xstate_def) |
13673 | 1242 |
done |
1243 |
||
1244 |
theorem compiler_correctness_exec: " |
|
22271 | 1245 |
\<lbrakk> G \<turnstile> Norm (hp, loc) -st-> Norm (hp', loc'); |
13673 | 1246 |
wf_java_prog G; |
1247 |
class_sig_defined G C S; |
|
1248 |
wtpd_stmt (env_of_jmb G C S) st; |
|
1249 |
(None,hp,loc) ::\<preceq> (env_of_jmb G C S) \<rbrakk> \<Longrightarrow> |
|
1250 |
{(TranslComp.comp G), C, S} \<turnstile> |
|
1251 |
{hp, os, (locvars_locals G C S loc)} |
|
1252 |
>- (compStmt (gmb G C S) st) \<rightarrow> |
|
1253 |
{hp', os, (locvars_locals G C S loc')}" |
|
1254 |
apply (frule compiler_correctness [THEN conjunct2 [THEN conjunct2]]) |
|
14045 | 1255 |
apply (auto simp: gh_def gx_def gs_def gl_def locvars_xstate_def) |
13673 | 1256 |
done |
1257 |
||
1258 |
(**********************************************************************) |
|
1259 |
||
1260 |
||
1261 |
(* reinstall pair splits *) |
|
1262 |
declare split_paired_All [simp] split_paired_Ex [simp] |
|
1263 |
||
14045 | 1264 |
declare wf_prog_ws_prog [simp del] |
1265 |
||
13673 | 1266 |
end |