| author | Andreas Lochbihler <mail@andreas-lochbihler.de> | 
| Sun, 31 Jan 2021 12:10:20 +0100 | |
| changeset 73213 | bb35f7f60d6c | 
| parent 67443 | 3abf6a722518 | 
| child 80914 | d97fdabd9e2b | 
| permissions | -rw-r--r-- | 
| 8011 | 1  | 
(* Title: HOL/MicroJava/J/Conform.thy  | 
2  | 
Author: David von Oheimb  | 
|
3  | 
Copyright 1999 Technische Universitaet Muenchen  | 
|
| 11070 | 4  | 
*)  | 
| 8011 | 5  | 
|
| 61361 | 6  | 
section \<open>Conformity Relations for Type Soundness Proof\<close>  | 
| 8011 | 7  | 
|
| 16417 | 8  | 
theory Conform imports State WellType Exceptions begin  | 
| 
9346
 
297dcbf64526
re-structuring MicroJava; added Example; corrected := syntax; simplfied cast
 
oheimb 
parents: 
8082 
diff
changeset
 | 
9  | 
|
| 
67443
 
3abf6a722518
standardized towards new-style formal comments: isabelle update_comments;
 
wenzelm 
parents: 
62042 
diff
changeset
 | 
10  | 
type_synonym 'c env' = "'c prog \<times> (vname \<rightharpoonup> ty)" \<comment> \<open>same as \<open>env\<close> of \<open>WellType.thy\<close>\<close>  | 
| 8011 | 11  | 
|
| 61994 | 12  | 
definition hext :: "aheap => aheap => bool" ("_ \<le>| _" [51,51] 50) where
 | 
13  | 
"h\<le>|h' == \<forall>a C fs. h a = Some(C,fs) --> (\<exists>fs'. h' a = Some(C,fs'))"  | 
|
| 8011 | 14  | 
|
| 
35416
 
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
 
haftmann 
parents: 
30235 
diff
changeset
 | 
15  | 
definition conf :: "'c prog => aheap => val => ty => bool"  | 
| 61994 | 16  | 
                                   ("_,_ \<turnstile> _ ::\<preceq> _"  [51,51,51,51] 50) where
 | 
17  | 
"G,h\<turnstile>v::\<preceq>T == \<exists>T'. typeof (map_option obj_ty o h) v = Some T' \<and> G\<turnstile>T'\<preceq>T"  | 
|
| 8011 | 18  | 
|
| 
35416
 
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
 
haftmann 
parents: 
30235 
diff
changeset
 | 
19  | 
definition lconf :: "'c prog => aheap => ('a \<rightharpoonup> val) => ('a \<rightharpoonup> ty) => bool"
 | 
| 61994 | 20  | 
                                   ("_,_ \<turnstile> _ [::\<preceq>] _" [51,51,51,51] 50) where
 | 
21  | 
"G,h\<turnstile>vs[::\<preceq>]Ts == \<forall>n T. Ts n = Some T --> (\<exists>v. vs n = Some v \<and> G,h\<turnstile>v::\<preceq>T)"  | 
|
| 8011 | 22  | 
|
| 61994 | 23  | 
definition oconf :: "'c prog => aheap => obj => bool" ("_,_ \<turnstile> _ \<surd>" [51,51,51] 50) where
 | 
24  | 
"G,h\<turnstile>obj \<surd> == G,h\<turnstile>snd obj[::\<preceq>]map_of (fields (G,fst obj))"  | 
|
| 8011 | 25  | 
|
| 61994 | 26  | 
definition hconf :: "'c prog => aheap => bool" ("_ \<turnstile>h _ \<surd>" [51,51] 50) where
 | 
27  | 
"G\<turnstile>h h \<surd> == \<forall>a obj. h a = Some obj --> G,h\<turnstile>obj \<surd>"  | 
|
| 13672 | 28  | 
|
| 
35416
 
d8d7d1b785af
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
 
haftmann 
parents: 
30235 
diff
changeset
 | 
29  | 
definition xconf :: "aheap \<Rightarrow> val option \<Rightarrow> bool" where  | 
| 13672 | 30  | 
"xconf hp vo == preallocated hp \<and> (\<forall> v. (vo = Some v) \<longrightarrow> (\<exists> xc. v = (Addr (XcptRef xc))))"  | 
| 8011 | 31  | 
|
| 61994 | 32  | 
definition conforms :: "xstate => java_mb env' => bool" ("_ ::\<preceq> _" [51,51] 50) where
 | 
33  | 
"s::\<preceq>E == prg E\<turnstile>h heap (store s) \<surd> \<and>  | 
|
34  | 
prg E,heap (store s)\<turnstile>locals (store s)[::\<preceq>]localT E \<and>  | 
|
| 13672 | 35  | 
xconf (heap (store s)) (abrupt s)"  | 
| 8011 | 36  | 
|
| 
10061
 
fe82134773dc
added HTML syntax; added spaces in normal syntax for better documents
 
kleing 
parents: 
10042 
diff
changeset
 | 
37  | 
|
| 58886 | 38  | 
subsection "hext"  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
39  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
40  | 
lemma hextI:  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
41  | 
" \<forall>a C fs . h a = Some (C,fs) -->  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
42  | 
(\<exists>fs'. h' a = Some (C,fs')) ==> h\<le>|h'"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
43  | 
apply (unfold hext_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
44  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
45  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
46  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
47  | 
lemma hext_objD: "[|h\<le>|h'; h a = Some (C,fs) |] ==> \<exists>fs'. h' a = Some (C,fs')"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
48  | 
apply (unfold hext_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
49  | 
apply (force)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
50  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
51  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
52  | 
lemma hext_refl [simp]: "h\<le>|h"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
53  | 
apply (rule hextI)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
54  | 
apply (fast)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
55  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
56  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
57  | 
lemma hext_new [simp]: "h a = None ==> h\<le>|h(a\<mapsto>x)"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
58  | 
apply (rule hextI)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
59  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
60  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
61  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
62  | 
lemma hext_trans: "[|h\<le>|h'; h'\<le>|h''|] ==> h\<le>|h''"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
63  | 
apply (rule hextI)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
64  | 
apply (fast dest: hext_objD)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
65  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
66  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
67  | 
lemma hext_upd_obj: "h a = Some (C,fs) ==> h\<le>|h(a\<mapsto>(C,fs'))"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
68  | 
apply (rule hextI)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
69  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
70  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
71  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
72  | 
|
| 58886 | 73  | 
subsection "conf"  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
74  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
75  | 
lemma conf_Null [simp]: "G,h\<turnstile>Null::\<preceq>T = G\<turnstile>RefT NullT\<preceq>T"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
76  | 
apply (unfold conf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
77  | 
apply (simp (no_asm))  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
78  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
79  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
80  | 
lemma conf_litval [rule_format (no_asm), simp]:  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
81  | 
"typeof (\<lambda>v. None) v = Some T --> G,h\<turnstile>v::\<preceq>T"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
82  | 
apply (unfold conf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
83  | 
apply (rule val.induct)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
84  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
85  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
86  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
87  | 
lemma conf_AddrI: "[|h a = Some obj; G\<turnstile>obj_ty obj\<preceq>T|] ==> G,h\<turnstile>Addr a::\<preceq>T"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
88  | 
apply (unfold conf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
89  | 
apply (simp)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
90  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
91  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
92  | 
lemma conf_obj_AddrI: "[|h a = Some (C,fs); G\<turnstile>C\<preceq>C D|] ==> G,h\<turnstile>Addr a::\<preceq> Class D"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
93  | 
apply (unfold conf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
94  | 
apply (simp)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
95  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
96  | 
|
| 12517 | 97  | 
lemma defval_conf [rule_format (no_asm)]:  | 
98  | 
"is_type G T --> G,h\<turnstile>default_val T::\<preceq>T"  | 
|
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
99  | 
apply (unfold conf_def)  | 
| 
14174
 
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
 
ballarin 
parents: 
14134 
diff
changeset
 | 
100  | 
apply (rule_tac y = "T" in ty.exhaust)  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
101  | 
apply (erule ssubst)  | 
| 58263 | 102  | 
apply (rename_tac prim_ty, rule_tac y = "prim_ty" in prim_ty.exhaust)  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
103  | 
apply (auto simp add: widen.null)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
104  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
105  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
106  | 
lemma conf_upd_obj:  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
107  | 
"h a = Some (C,fs) ==> (G,h(a\<mapsto>(C,fs'))\<turnstile>x::\<preceq>T) = (G,h\<turnstile>x::\<preceq>T)"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
108  | 
apply (unfold conf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
109  | 
apply (rule val.induct)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
110  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
111  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
112  | 
|
| 12517 | 113  | 
lemma conf_widen [rule_format (no_asm)]:  | 
114  | 
"wf_prog wf_mb G ==> G,h\<turnstile>x::\<preceq>T --> G\<turnstile>T\<preceq>T' --> G,h\<turnstile>x::\<preceq>T'"  | 
|
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
115  | 
apply (unfold conf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
116  | 
apply (rule val.induct)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
117  | 
apply (auto intro: widen_trans)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
118  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
119  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
120  | 
lemma conf_hext [rule_format (no_asm)]: "h\<le>|h' ==> G,h\<turnstile>v::\<preceq>T --> G,h'\<turnstile>v::\<preceq>T"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
121  | 
apply (unfold conf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
122  | 
apply (rule val.induct)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
123  | 
apply (auto dest: hext_objD)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
124  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
125  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
126  | 
lemma new_locD: "[|h a = None; G,h\<turnstile>Addr t::\<preceq>T|] ==> t\<noteq>a"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
127  | 
apply (unfold conf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
128  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
129  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
130  | 
|
| 52847 | 131  | 
lemma conf_RefTD [rule_format]:  | 
132  | 
"G,h\<turnstile>a'::\<preceq>RefT T \<Longrightarrow> a' = Null \<or>  | 
|
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
133  | 
(\<exists>a obj T'. a' = Addr a \<and> h a = Some obj \<and> obj_ty obj = T' \<and> G\<turnstile>T'\<preceq>RefT T)"  | 
| 52847 | 134  | 
unfolding conf_def by (induct a') auto  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
135  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
136  | 
lemma conf_NullTD: "G,h\<turnstile>a'::\<preceq>RefT NullT ==> a' = Null"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
137  | 
apply (drule conf_RefTD)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
138  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
139  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
140  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
141  | 
lemma non_npD: "[|a' \<noteq> Null; G,h\<turnstile>a'::\<preceq>RefT t|] ==>  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
142  | 
\<exists>a C fs. a' = Addr a \<and> h a = Some (C,fs) \<and> G\<turnstile>Class C\<preceq>RefT t"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
143  | 
apply (drule conf_RefTD)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
144  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
145  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
146  | 
|
| 12951 | 147  | 
lemma non_np_objD: "!!G. [|a' \<noteq> Null; G,h\<turnstile>a'::\<preceq> Class C|] ==>  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
148  | 
(\<exists>a C' fs. a' = Addr a \<and> h a = Some (C',fs) \<and> G\<turnstile>C'\<preceq>C C)"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
149  | 
apply (fast dest: non_npD)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
150  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
151  | 
|
| 12517 | 152  | 
lemma non_np_objD' [rule_format (no_asm)]:  | 
153  | 
"a' \<noteq> Null ==> wf_prog wf_mb G ==> G,h\<turnstile>a'::\<preceq>RefT t -->  | 
|
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
154  | 
(\<exists>a C fs. a' = Addr a \<and> h a = Some (C,fs) \<and> G\<turnstile>Class C\<preceq>RefT t)"  | 
| 
14174
 
f3cafd2929d5
Methods rule_tac etc support static (Isar) contexts.
 
ballarin 
parents: 
14134 
diff
changeset
 | 
155  | 
apply(rule_tac y = "t" in ref_ty.exhaust)  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
156  | 
apply (fast dest: conf_NullTD)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
157  | 
apply (fast dest: non_np_objD)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
158  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
159  | 
|
| 12517 | 160  | 
lemma conf_list_gext_widen [rule_format (no_asm)]:  | 
161  | 
"wf_prog wf_mb G ==> \<forall>Ts Ts'. list_all2 (conf G h) vs Ts -->  | 
|
162  | 
list_all2 (\<lambda>T T'. G\<turnstile>T\<preceq>T') Ts Ts' --> list_all2 (conf G h) vs Ts'"  | 
|
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
163  | 
apply(induct_tac "vs")  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
164  | 
apply(clarsimp)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
165  | 
apply(clarsimp)  | 
| 59199 | 166  | 
apply(frule list_all2_lengthD [symmetric])  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
167  | 
apply(simp (no_asm_use) add: length_Suc_conv)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
168  | 
apply(safe)  | 
| 59199 | 169  | 
apply(frule list_all2_lengthD [symmetric])  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
170  | 
apply(simp (no_asm_use) add: length_Suc_conv)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
171  | 
apply(clarify)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
172  | 
apply(fast elim: conf_widen)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
173  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
174  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
175  | 
|
| 58886 | 176  | 
subsection "lconf"  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
177  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
178  | 
lemma lconfD: "[| G,h\<turnstile>vs[::\<preceq>]Ts; Ts n = Some T |] ==> G,h\<turnstile>(the (vs n))::\<preceq>T"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
179  | 
apply (unfold lconf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
180  | 
apply (force)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
181  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
182  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
183  | 
lemma lconf_hext [elim]: "[| G,h\<turnstile>l[::\<preceq>]L; h\<le>|h' |] ==> G,h'\<turnstile>l[::\<preceq>]L"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
184  | 
apply (unfold lconf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
185  | 
apply (fast elim: conf_hext)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
186  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
187  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
188  | 
lemma lconf_upd: "!!X. [| G,h\<turnstile>l[::\<preceq>]lT;  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
189  | 
G,h\<turnstile>v::\<preceq>T; lT va = Some T |] ==> G,h\<turnstile>l(va\<mapsto>v)[::\<preceq>]lT"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
190  | 
apply (unfold lconf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
191  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
192  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
193  | 
|
| 12517 | 194  | 
lemma lconf_init_vars_lemma [rule_format (no_asm)]:  | 
195  | 
"\<forall>x. P x --> R (dv x) x ==> (\<forall>x. map_of fs f = Some x --> P x) -->  | 
|
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
196  | 
(\<forall>T. map_of fs f = Some T -->  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
197  | 
(\<exists>v. map_of (map (\<lambda>(f,ft). (f, dv ft)) fs) f = Some v \<and> R v T))"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
198  | 
apply( induct_tac "fs")  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
199  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
200  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
201  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
202  | 
lemma lconf_init_vars [intro!]:  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
203  | 
"\<forall>n. \<forall>T. map_of fs n = Some T --> is_type G T ==> G,h\<turnstile>init_vars fs[::\<preceq>]map_of fs"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
204  | 
apply (unfold lconf_def init_vars_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
205  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
206  | 
apply( rule lconf_init_vars_lemma)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
207  | 
apply( erule_tac [3] asm_rl)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
208  | 
apply( intro strip)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
209  | 
apply( erule defval_conf)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
210  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
211  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
212  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
213  | 
lemma lconf_ext: "[|G,s\<turnstile>l[::\<preceq>]L; G,s\<turnstile>v::\<preceq>T|] ==> G,s\<turnstile>l(vn\<mapsto>v)[::\<preceq>]L(vn\<mapsto>T)"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
214  | 
apply (unfold lconf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
215  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
216  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
217  | 
|
| 12517 | 218  | 
lemma lconf_ext_list [rule_format (no_asm)]:  | 
| 12888 | 219  | 
"G,h\<turnstile>l[::\<preceq>]L ==> \<forall>vs Ts. distinct vns --> length Ts = length vns -->  | 
| 12517 | 220  | 
list_all2 (\<lambda>v T. G,h\<turnstile>v::\<preceq>T) vs Ts --> G,h\<turnstile>l(vns[\<mapsto>]vs)[::\<preceq>]L(vns[\<mapsto>]Ts)"  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
221  | 
apply (unfold lconf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
222  | 
apply( induct_tac "vns")  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
223  | 
apply( clarsimp)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
224  | 
apply( clarsimp)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
225  | 
apply( frule list_all2_lengthD)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
226  | 
apply( auto simp add: length_Suc_conv)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
227  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
228  | 
|
| 13672 | 229  | 
lemma lconf_restr: "\<lbrakk>lT vn = None; G, h \<turnstile> l [::\<preceq>] lT(vn\<mapsto>T)\<rbrakk> \<Longrightarrow> G, h \<turnstile> l [::\<preceq>] lT"  | 
230  | 
apply (unfold lconf_def)  | 
|
231  | 
apply (intro strip)  | 
|
232  | 
apply (case_tac "n = vn")  | 
|
233  | 
apply auto  | 
|
234  | 
done  | 
|
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
235  | 
|
| 58886 | 236  | 
subsection "oconf"  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
237  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
238  | 
lemma oconf_hext: "G,h\<turnstile>obj\<surd> ==> h\<le>|h' ==> G,h'\<turnstile>obj\<surd>"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
239  | 
apply (unfold oconf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
240  | 
apply (fast)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
241  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
242  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
243  | 
lemma oconf_obj: "G,h\<turnstile>(C,fs)\<surd> =  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
244  | 
(\<forall>T f. map_of(fields (G,C)) f = Some T --> (\<exists>v. fs f = Some v \<and> G,h\<turnstile>v::\<preceq>T))"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
245  | 
apply (unfold oconf_def lconf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
246  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
247  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
248  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
249  | 
lemmas oconf_objD = oconf_obj [THEN iffD1, THEN spec, THEN spec, THEN mp]  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
250  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
251  | 
|
| 58886 | 252  | 
subsection "hconf"  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
253  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
254  | 
lemma hconfD: "[|G\<turnstile>h h\<surd>; h a = Some obj|] ==> G,h\<turnstile>obj\<surd>"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
255  | 
apply (unfold hconf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
256  | 
apply (fast)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
257  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
258  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
259  | 
lemma hconfI: "\<forall>a obj. h a=Some obj --> G,h\<turnstile>obj\<surd> ==> G\<turnstile>h h\<surd>"  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
260  | 
apply (unfold hconf_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
261  | 
apply (fast)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
262  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
263  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
264  | 
|
| 58886 | 265  | 
subsection "xconf"  | 
| 13672 | 266  | 
|
267  | 
lemma xconf_raise_if: "xconf h x \<Longrightarrow> xconf h (raise_if b xcn x)"  | 
|
268  | 
by (simp add: xconf_def raise_if_def)  | 
|
269  | 
||
270  | 
||
271  | 
||
| 58886 | 272  | 
subsection "conforms"  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
273  | 
|
| 13672 | 274  | 
lemma conforms_heapD: "(x, (h, l))::\<preceq>(G, lT) ==> G\<turnstile>h h\<surd>"  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
275  | 
apply (unfold conforms_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
276  | 
apply (simp)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
277  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
278  | 
|
| 13672 | 279  | 
lemma conforms_localD: "(x, (h, l))::\<preceq>(G, lT) ==> G,h\<turnstile>l[::\<preceq>]lT"  | 
280  | 
apply (unfold conforms_def)  | 
|
281  | 
apply (simp)  | 
|
282  | 
done  | 
|
283  | 
||
284  | 
lemma conforms_xcptD: "(x, (h, l))::\<preceq>(G, lT) ==> xconf h x"  | 
|
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
285  | 
apply (unfold conforms_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
286  | 
apply (simp)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
287  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
288  | 
|
| 13672 | 289  | 
lemma conformsI: "[|G\<turnstile>h h\<surd>; G,h\<turnstile>l[::\<preceq>]lT; xconf h x|] ==> (x, (h, l))::\<preceq>(G, lT)"  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
290  | 
apply (unfold conforms_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
291  | 
apply auto  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
292  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
293  | 
|
| 13672 | 294  | 
lemma conforms_restr: "\<lbrakk>lT vn = None; s ::\<preceq> (G, lT(vn\<mapsto>T)) \<rbrakk> \<Longrightarrow> s ::\<preceq> (G, lT)"  | 
295  | 
by (simp add: conforms_def, fast intro: lconf_restr)  | 
|
296  | 
||
297  | 
lemma conforms_xcpt_change: "\<lbrakk> (x, (h,l))::\<preceq> (G, lT); xconf h x \<longrightarrow> xconf h x' \<rbrakk> \<Longrightarrow> (x', (h,l))::\<preceq> (G, lT)"  | 
|
298  | 
by (simp add: conforms_def)  | 
|
299  | 
||
300  | 
||
301  | 
lemma preallocated_hext: "\<lbrakk> preallocated h; h\<le>|h'\<rbrakk> \<Longrightarrow> preallocated h'"  | 
|
302  | 
by (simp add: preallocated_def hext_def)  | 
|
303  | 
||
304  | 
lemma xconf_hext: "\<lbrakk> xconf h vo; h\<le>|h'\<rbrakk> \<Longrightarrow> xconf h' vo"  | 
|
305  | 
by (simp add: xconf_def preallocated_def hext_def)  | 
|
306  | 
||
307  | 
lemma conforms_hext: "[|(x,(h,l))::\<preceq>(G,lT); h\<le>|h'; G\<turnstile>h h'\<surd> |]  | 
|
308  | 
==> (x,(h',l))::\<preceq>(G,lT)"  | 
|
| 52847 | 309  | 
by (fast dest: conforms_localD conforms_xcptD elim!: conformsI xconf_hext)  | 
| 13672 | 310  | 
|
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
311  | 
|
| 12517 | 312  | 
lemma conforms_upd_obj:  | 
| 13672 | 313  | 
"[|(x,(h,l))::\<preceq>(G, lT); G,h(a\<mapsto>obj)\<turnstile>obj\<surd>; h\<le>|h(a\<mapsto>obj)|]  | 
314  | 
==> (x,(h(a\<mapsto>obj),l))::\<preceq>(G, lT)"  | 
|
| 12517 | 315  | 
apply(rule conforms_hext)  | 
316  | 
apply auto  | 
|
317  | 
apply(rule hconfI)  | 
|
318  | 
apply(drule conforms_heapD)  | 
|
| 46206 | 319  | 
apply(auto elim: oconf_hext dest: hconfD)  | 
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
320  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
321  | 
|
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
322  | 
lemma conforms_upd_local:  | 
| 13672 | 323  | 
"[|(x,(h, l))::\<preceq>(G, lT); G,h\<turnstile>v::\<preceq>T; lT va = Some T|]  | 
324  | 
==> (x,(h, l(va\<mapsto>v)))::\<preceq>(G, lT)"  | 
|
| 
11026
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
325  | 
apply (unfold conforms_def)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
326  | 
apply( auto elim: lconf_upd)  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
327  | 
done  | 
| 
 
a50365d21144
converted to Isar, simplifying recursion on class hierarchy
 
oheimb 
parents: 
10061 
diff
changeset
 | 
328  | 
|
| 8011 | 329  | 
end  |