author | wenzelm |
Fri, 22 Apr 2011 13:58:13 +0200 | |
changeset 42455 | 6702c984bf5a |
parent 40671 | 5e46057ba8e0 |
child 48073 | 1b609a7837ef |
permissions | -rw-r--r-- |
31870 | 1 |
(* Title: HOL/Imperative_HOL/Array.thy |
26170 | 2 |
Author: John Matthews, Galois Connections; Alexander Krauss, Lukas Bulwahn & Florian Haftmann, TU Muenchen |
3 |
*) |
|
4 |
||
5 |
header {* Monadic arrays *} |
|
6 |
||
7 |
theory Array |
|
31203
5c8fb4fd67e0
moved Code_Index, Random and Quickcheck before Main
haftmann
parents:
29822
diff
changeset
|
8 |
imports Heap_Monad |
26170 | 9 |
begin |
10 |
||
37752 | 11 |
subsection {* Primitives *} |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
12 |
|
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
13 |
definition present :: "heap \<Rightarrow> 'a\<Colon>heap array \<Rightarrow> bool" where |
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
14 |
"present h a \<longleftrightarrow> addr_of_array a < lim h" |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
15 |
|
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
16 |
definition get :: "heap \<Rightarrow> 'a\<Colon>heap array \<Rightarrow> 'a list" where |
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
17 |
"get h a = map from_nat (arrays h (TYPEREP('a)) (addr_of_array a))" |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
18 |
|
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
19 |
definition set :: "'a\<Colon>heap array \<Rightarrow> 'a list \<Rightarrow> heap \<Rightarrow> heap" where |
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
20 |
"set a x = arrays_update (\<lambda>h. h(TYPEREP('a) := ((h(TYPEREP('a))) (addr_of_array a:=map to_nat x))))" |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
21 |
|
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
22 |
definition alloc :: "'a list \<Rightarrow> heap \<Rightarrow> 'a\<Colon>heap array \<times> heap" where |
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
23 |
"alloc xs h = (let |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
24 |
l = lim h; |
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
25 |
r = Array l; |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
26 |
h'' = set r xs (h\<lparr>lim := l + 1\<rparr>) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
27 |
in (r, h''))" |
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
28 |
|
37802 | 29 |
definition length :: "heap \<Rightarrow> 'a\<Colon>heap array \<Rightarrow> nat" where |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
30 |
"length h a = List.length (get h a)" |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
31 |
|
37798
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
32 |
definition update :: "'a\<Colon>heap array \<Rightarrow> nat \<Rightarrow> 'a \<Rightarrow> heap \<Rightarrow> heap" where |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
33 |
"update a i x h = set a ((get h a)[i:=x]) h" |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
34 |
|
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
35 |
definition noteq :: "'a\<Colon>heap array \<Rightarrow> 'b\<Colon>heap array \<Rightarrow> bool" (infix "=!!=" 70) where |
37752 | 36 |
"r =!!= s \<longleftrightarrow> TYPEREP('a) \<noteq> TYPEREP('b) \<or> addr_of_array r \<noteq> addr_of_array s" |
37 |
||
38 |
||
39 |
subsection {* Monad operations *} |
|
40 |
||
41 |
definition new :: "nat \<Rightarrow> 'a\<Colon>heap \<Rightarrow> 'a array Heap" where |
|
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
42 |
[code del]: "new n x = Heap_Monad.heap (alloc (replicate n x))" |
37752 | 43 |
|
44 |
definition of_list :: "'a\<Colon>heap list \<Rightarrow> 'a array Heap" where |
|
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
45 |
[code del]: "of_list xs = Heap_Monad.heap (alloc xs)" |
37752 | 46 |
|
47 |
definition make :: "nat \<Rightarrow> (nat \<Rightarrow> 'a\<Colon>heap) \<Rightarrow> 'a array Heap" where |
|
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
48 |
[code del]: "make n f = Heap_Monad.heap (alloc (map f [0 ..< n]))" |
37752 | 49 |
|
50 |
definition len :: "'a\<Colon>heap array \<Rightarrow> nat Heap" where |
|
37802 | 51 |
[code del]: "len a = Heap_Monad.tap (\<lambda>h. length h a)" |
37752 | 52 |
|
53 |
definition nth :: "'a\<Colon>heap array \<Rightarrow> nat \<Rightarrow> 'a Heap" where |
|
37802 | 54 |
[code del]: "nth a i = Heap_Monad.guard (\<lambda>h. i < length h a) |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
55 |
(\<lambda>h. (get h a ! i, h))" |
37752 | 56 |
|
57 |
definition upd :: "nat \<Rightarrow> 'a \<Rightarrow> 'a\<Colon>heap array \<Rightarrow> 'a\<Colon>heap array Heap" where |
|
37802 | 58 |
[code del]: "upd i x a = Heap_Monad.guard (\<lambda>h. i < length h a) |
37798
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
59 |
(\<lambda>h. (a, update a i x h))" |
37752 | 60 |
|
61 |
definition map_entry :: "nat \<Rightarrow> ('a\<Colon>heap \<Rightarrow> 'a) \<Rightarrow> 'a array \<Rightarrow> 'a array Heap" where |
|
37802 | 62 |
[code del]: "map_entry i f a = Heap_Monad.guard (\<lambda>h. i < length h a) |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
63 |
(\<lambda>h. (a, update a i (f (get h a ! i)) h))" |
37752 | 64 |
|
65 |
definition swap :: "nat \<Rightarrow> 'a \<Rightarrow> 'a\<Colon>heap array \<Rightarrow> 'a Heap" where |
|
37802 | 66 |
[code del]: "swap i x a = Heap_Monad.guard (\<lambda>h. i < length h a) |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
67 |
(\<lambda>h. (get h a ! i, update a i x h))" |
37752 | 68 |
|
69 |
definition freeze :: "'a\<Colon>heap array \<Rightarrow> 'a list Heap" where |
|
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
70 |
[code del]: "freeze a = Heap_Monad.tap (\<lambda>h. get h a)" |
37752 | 71 |
|
72 |
||
73 |
subsection {* Properties *} |
|
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
74 |
|
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
75 |
text {* FIXME: Does there exist a "canonical" array axiomatisation in |
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
76 |
the literature? *} |
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
77 |
|
37758 | 78 |
text {* Primitives *} |
79 |
||
37807 | 80 |
lemma noteq_sym: "a =!!= b \<Longrightarrow> b =!!= a" |
81 |
and unequal [simp]: "a \<noteq> a' \<longleftrightarrow> a =!!= a'" |
|
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
82 |
unfolding noteq_def by auto |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
83 |
|
37807 | 84 |
lemma noteq_irrefl: "r =!!= r \<Longrightarrow> False" |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
85 |
unfolding noteq_def by auto |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
86 |
|
37807 | 87 |
lemma present_alloc_noteq: "present h a \<Longrightarrow> a =!!= fst (alloc xs h)" |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
88 |
by (simp add: present_def noteq_def alloc_def Let_def) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
89 |
|
37807 | 90 |
lemma get_set_eq [simp]: "get (set r x h) r = x" |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
91 |
by (simp add: get_def set_def o_def) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
92 |
|
37807 | 93 |
lemma get_set_neq [simp]: "r =!!= s \<Longrightarrow> get (set s x h) r = get h r" |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
94 |
by (simp add: noteq_def get_def set_def) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
95 |
|
37807 | 96 |
lemma set_same [simp]: |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
97 |
"set r x (set r y h) = set r x h" |
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
98 |
by (simp add: set_def) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
99 |
|
37807 | 100 |
lemma set_set_swap: |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
101 |
"r =!!= r' \<Longrightarrow> set r x (set r' x' h) = set r' x' (set r x h)" |
39302
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
nipkow
parents:
39198
diff
changeset
|
102 |
by (simp add: Let_def fun_eq_iff noteq_def set_def) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
103 |
|
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
104 |
lemma get_update_eq [simp]: |
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
105 |
"get (update a i v h) a = (get h a) [i := v]" |
37798
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
106 |
by (simp add: update_def) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
107 |
|
37807 | 108 |
lemma nth_update_neq [simp]: |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
109 |
"a =!!= b \<Longrightarrow> get (update b j v h) a ! i = get h a ! i" |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
110 |
by (simp add: update_def noteq_def) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
111 |
|
37807 | 112 |
lemma get_update_elem_neqIndex [simp]: |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
113 |
"i \<noteq> j \<Longrightarrow> get (update a j v h) a ! i = get h a ! i" |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
114 |
by simp |
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
115 |
|
37798
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
116 |
lemma length_update [simp]: |
37802 | 117 |
"length (update b i v h) = length h" |
39302
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
nipkow
parents:
39198
diff
changeset
|
118 |
by (simp add: update_def length_def set_def get_def fun_eq_iff) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
119 |
|
37807 | 120 |
lemma update_swap_neq: |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
121 |
"a =!!= a' \<Longrightarrow> |
37798
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
122 |
update a i v (update a' i' v' h) |
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
123 |
= update a' i' v' (update a i v h)" |
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
124 |
apply (unfold update_def) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
125 |
apply simp |
37807 | 126 |
apply (subst set_set_swap, assumption) |
127 |
apply (subst get_set_neq) |
|
128 |
apply (erule noteq_sym) |
|
129 |
apply simp |
|
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
130 |
done |
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
131 |
|
37798
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
132 |
lemma update_swap_neqIndex: |
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
133 |
"\<lbrakk> i \<noteq> i' \<rbrakk> \<Longrightarrow> update a i v (update a i' v' h) = update a i' v' (update a i v h)" |
37807 | 134 |
by (auto simp add: update_def set_set_swap list_update_swap) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
135 |
|
37807 | 136 |
lemma get_alloc: |
40360 | 137 |
"get (snd (alloc xs h)) (fst (alloc ys h)) = xs" |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
138 |
by (simp add: Let_def split_def alloc_def) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
139 |
|
40360 | 140 |
lemma length_alloc: |
141 |
"length (snd (alloc (xs :: 'a::heap list) h)) (fst (alloc (ys :: 'a list) h)) = List.length xs" |
|
142 |
by (simp add: Array.length_def get_alloc) |
|
143 |
||
37807 | 144 |
lemma set: |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
145 |
"set (fst (alloc ls h)) |
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
146 |
new_ls (snd (alloc ls h)) |
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
147 |
= snd (alloc new_ls h)" |
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
148 |
by (simp add: Let_def split_def alloc_def) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
149 |
|
37807 | 150 |
lemma present_update [simp]: |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
151 |
"present (update b i v h) = present h" |
39302
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
nipkow
parents:
39198
diff
changeset
|
152 |
by (simp add: update_def present_def set_def get_def fun_eq_iff) |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
153 |
|
37807 | 154 |
lemma present_alloc [simp]: |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
155 |
"present (snd (alloc xs h)) (fst (alloc xs h))" |
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
156 |
by (simp add: present_def alloc_def set_def Let_def) |
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
157 |
|
37807 | 158 |
lemma not_present_alloc [simp]: |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
159 |
"\<not> present h (fst (alloc xs h))" |
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
160 |
by (simp add: present_def alloc_def Let_def) |
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
161 |
|
37758 | 162 |
|
163 |
text {* Monad operations *} |
|
164 |
||
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
165 |
lemma execute_new [execute_simps]: |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
166 |
"execute (new n x) h = Some (alloc (replicate n x) h)" |
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
167 |
by (simp add: new_def execute_simps) |
37758 | 168 |
|
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
169 |
lemma success_newI [success_intros]: |
37758 | 170 |
"success (new n x) h" |
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
171 |
by (auto intro: success_intros simp add: new_def) |
26170 | 172 |
|
40671 | 173 |
lemma effect_newI [effect_intros]: |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
174 |
assumes "(a, h') = alloc (replicate n x) h" |
40671 | 175 |
shows "effect (new n x) h h' a" |
176 |
by (rule effectI) (simp add: assms execute_simps) |
|
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
177 |
|
40671 | 178 |
lemma effect_newE [effect_elims]: |
179 |
assumes "effect (new n x) h h' r" |
|
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
180 |
obtains "r = fst (alloc (replicate n x) h)" "h' = snd (alloc (replicate n x) h)" |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
181 |
"get h' r = replicate n x" "present h' r" "\<not> present h r" |
40671 | 182 |
using assms by (rule effectE) (simp add: get_alloc execute_simps) |
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
183 |
|
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
184 |
lemma execute_of_list [execute_simps]: |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
185 |
"execute (of_list xs) h = Some (alloc xs h)" |
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
186 |
by (simp add: of_list_def execute_simps) |
37758 | 187 |
|
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
188 |
lemma success_of_listI [success_intros]: |
37758 | 189 |
"success (of_list xs) h" |
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
190 |
by (auto intro: success_intros simp add: of_list_def) |
26170 | 191 |
|
40671 | 192 |
lemma effect_of_listI [effect_intros]: |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
193 |
assumes "(a, h') = alloc xs h" |
40671 | 194 |
shows "effect (of_list xs) h h' a" |
195 |
by (rule effectI) (simp add: assms execute_simps) |
|
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
196 |
|
40671 | 197 |
lemma effect_of_listE [effect_elims]: |
198 |
assumes "effect (of_list xs) h h' r" |
|
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
199 |
obtains "r = fst (alloc xs h)" "h' = snd (alloc xs h)" |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
200 |
"get h' r = xs" "present h' r" "\<not> present h r" |
40671 | 201 |
using assms by (rule effectE) (simp add: get_alloc execute_simps) |
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
202 |
|
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
203 |
lemma execute_make [execute_simps]: |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
204 |
"execute (make n f) h = Some (alloc (map f [0 ..< n]) h)" |
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
205 |
by (simp add: make_def execute_simps) |
26170 | 206 |
|
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
207 |
lemma success_makeI [success_intros]: |
37758 | 208 |
"success (make n f) h" |
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
209 |
by (auto intro: success_intros simp add: make_def) |
37758 | 210 |
|
40671 | 211 |
lemma effect_makeI [effect_intros]: |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
212 |
assumes "(a, h') = alloc (map f [0 ..< n]) h" |
40671 | 213 |
shows "effect (make n f) h h' a" |
214 |
by (rule effectI) (simp add: assms execute_simps) |
|
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
215 |
|
40671 | 216 |
lemma effect_makeE [effect_elims]: |
217 |
assumes "effect (make n f) h h' r" |
|
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
218 |
obtains "r = fst (alloc (map f [0 ..< n]) h)" "h' = snd (alloc (map f [0 ..< n]) h)" |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
219 |
"get h' r = map f [0 ..< n]" "present h' r" "\<not> present h r" |
40671 | 220 |
using assms by (rule effectE) (simp add: get_alloc execute_simps) |
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
221 |
|
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
222 |
lemma execute_len [execute_simps]: |
37802 | 223 |
"execute (len a) h = Some (length h a, h)" |
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
224 |
by (simp add: len_def execute_simps) |
37758 | 225 |
|
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
226 |
lemma success_lenI [success_intros]: |
37758 | 227 |
"success (len a) h" |
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
228 |
by (auto intro: success_intros simp add: len_def) |
37752 | 229 |
|
40671 | 230 |
lemma effect_lengthI [effect_intros]: |
37802 | 231 |
assumes "h' = h" "r = length h a" |
40671 | 232 |
shows "effect (len a) h h' r" |
233 |
by (rule effectI) (simp add: assms execute_simps) |
|
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
234 |
|
40671 | 235 |
lemma effect_lengthE [effect_elims]: |
236 |
assumes "effect (len a) h h' r" |
|
37802 | 237 |
obtains "r = length h' a" "h' = h" |
40671 | 238 |
using assms by (rule effectE) (simp add: execute_simps) |
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
239 |
|
37758 | 240 |
lemma execute_nth [execute_simps]: |
37802 | 241 |
"i < length h a \<Longrightarrow> |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
242 |
execute (nth a i) h = Some (get h a ! i, h)" |
37802 | 243 |
"i \<ge> length h a \<Longrightarrow> execute (nth a i) h = None" |
37758 | 244 |
by (simp_all add: nth_def execute_simps) |
245 |
||
246 |
lemma success_nthI [success_intros]: |
|
37802 | 247 |
"i < length h a \<Longrightarrow> success (nth a i) h" |
37758 | 248 |
by (auto intro: success_intros simp add: nth_def) |
26170 | 249 |
|
40671 | 250 |
lemma effect_nthI [effect_intros]: |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
251 |
assumes "i < length h a" "h' = h" "r = get h a ! i" |
40671 | 252 |
shows "effect (nth a i) h h' r" |
253 |
by (rule effectI) (insert assms, simp add: execute_simps) |
|
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
254 |
|
40671 | 255 |
lemma effect_nthE [effect_elims]: |
256 |
assumes "effect (nth a i) h h' r" |
|
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
257 |
obtains "i < length h a" "r = get h a ! i" "h' = h" |
40671 | 258 |
using assms by (rule effectE) |
37802 | 259 |
(erule successE, cases "i < length h a", simp_all add: execute_simps) |
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
260 |
|
37758 | 261 |
lemma execute_upd [execute_simps]: |
37802 | 262 |
"i < length h a \<Longrightarrow> |
37798
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
263 |
execute (upd i x a) h = Some (a, update a i x h)" |
37802 | 264 |
"i \<ge> length h a \<Longrightarrow> execute (upd i x a) h = None" |
37758 | 265 |
by (simp_all add: upd_def execute_simps) |
26170 | 266 |
|
37758 | 267 |
lemma success_updI [success_intros]: |
37802 | 268 |
"i < length h a \<Longrightarrow> success (upd i x a) h" |
37758 | 269 |
by (auto intro: success_intros simp add: upd_def) |
270 |
||
40671 | 271 |
lemma effect_updI [effect_intros]: |
37802 | 272 |
assumes "i < length h a" "h' = update a i v h" |
40671 | 273 |
shows "effect (upd i v a) h h' a" |
274 |
by (rule effectI) (insert assms, simp add: execute_simps) |
|
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
275 |
|
40671 | 276 |
lemma effect_updE [effect_elims]: |
277 |
assumes "effect (upd i v a) h h' r" |
|
37802 | 278 |
obtains "r = a" "h' = update a i v h" "i < length h a" |
40671 | 279 |
using assms by (rule effectE) |
37802 | 280 |
(erule successE, cases "i < length h a", simp_all add: execute_simps) |
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
281 |
|
37758 | 282 |
lemma execute_map_entry [execute_simps]: |
37802 | 283 |
"i < length h a \<Longrightarrow> |
37758 | 284 |
execute (map_entry i f a) h = |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
285 |
Some (a, update a i (f (get h a ! i)) h)" |
37802 | 286 |
"i \<ge> length h a \<Longrightarrow> execute (map_entry i f a) h = None" |
37758 | 287 |
by (simp_all add: map_entry_def execute_simps) |
37752 | 288 |
|
37758 | 289 |
lemma success_map_entryI [success_intros]: |
37802 | 290 |
"i < length h a \<Longrightarrow> success (map_entry i f a) h" |
37758 | 291 |
by (auto intro: success_intros simp add: map_entry_def) |
292 |
||
40671 | 293 |
lemma effect_map_entryI [effect_intros]: |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
294 |
assumes "i < length h a" "h' = update a i (f (get h a ! i)) h" "r = a" |
40671 | 295 |
shows "effect (map_entry i f a) h h' r" |
296 |
by (rule effectI) (insert assms, simp add: execute_simps) |
|
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
297 |
|
40671 | 298 |
lemma effect_map_entryE [effect_elims]: |
299 |
assumes "effect (map_entry i f a) h h' r" |
|
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
300 |
obtains "r = a" "h' = update a i (f (get h a ! i)) h" "i < length h a" |
40671 | 301 |
using assms by (rule effectE) |
37802 | 302 |
(erule successE, cases "i < length h a", simp_all add: execute_simps) |
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
303 |
|
37758 | 304 |
lemma execute_swap [execute_simps]: |
37802 | 305 |
"i < length h a \<Longrightarrow> |
37758 | 306 |
execute (swap i x a) h = |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
307 |
Some (get h a ! i, update a i x h)" |
37802 | 308 |
"i \<ge> length h a \<Longrightarrow> execute (swap i x a) h = None" |
37758 | 309 |
by (simp_all add: swap_def execute_simps) |
310 |
||
311 |
lemma success_swapI [success_intros]: |
|
37802 | 312 |
"i < length h a \<Longrightarrow> success (swap i x a) h" |
37758 | 313 |
by (auto intro: success_intros simp add: swap_def) |
37752 | 314 |
|
40671 | 315 |
lemma effect_swapI [effect_intros]: |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
316 |
assumes "i < length h a" "h' = update a i x h" "r = get h a ! i" |
40671 | 317 |
shows "effect (swap i x a) h h' r" |
318 |
by (rule effectI) (insert assms, simp add: execute_simps) |
|
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
319 |
|
40671 | 320 |
lemma effect_swapE [effect_elims]: |
321 |
assumes "effect (swap i x a) h h' r" |
|
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
322 |
obtains "r = get h a ! i" "h' = update a i x h" "i < length h a" |
40671 | 323 |
using assms by (rule effectE) |
37802 | 324 |
(erule successE, cases "i < length h a", simp_all add: execute_simps) |
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
325 |
|
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
326 |
lemma execute_freeze [execute_simps]: |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
327 |
"execute (freeze a) h = Some (get h a, h)" |
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
328 |
by (simp add: freeze_def execute_simps) |
37758 | 329 |
|
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
330 |
lemma success_freezeI [success_intros]: |
37758 | 331 |
"success (freeze a) h" |
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
332 |
by (auto intro: success_intros simp add: freeze_def) |
26170 | 333 |
|
40671 | 334 |
lemma effect_freezeI [effect_intros]: |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
335 |
assumes "h' = h" "r = get h a" |
40671 | 336 |
shows "effect (freeze a) h h' r" |
337 |
by (rule effectI) (insert assms, simp add: execute_simps) |
|
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
338 |
|
40671 | 339 |
lemma effect_freezeE [effect_elims]: |
340 |
assumes "effect (freeze a) h h' r" |
|
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
341 |
obtains "h' = h" "r = get h a" |
40671 | 342 |
using assms by (rule effectE) (simp add: execute_simps) |
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
37758
diff
changeset
|
343 |
|
26170 | 344 |
lemma upd_return: |
345 |
"upd i x a \<guillemotright> return a = upd i x a" |
|
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
346 |
by (rule Heap_eqI) (simp add: bind_def guard_def upd_def execute_simps) |
26170 | 347 |
|
37752 | 348 |
lemma array_make: |
349 |
"new n x = make n (\<lambda>_. x)" |
|
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
350 |
by (rule Heap_eqI) (simp add: map_replicate_trivial execute_simps) |
26170 | 351 |
|
37845
b70d7a347964
first roughly working version of Imperative HOL for Scala
haftmann
parents:
37842
diff
changeset
|
352 |
lemma array_of_list_make [code]: |
37752 | 353 |
"of_list xs = make (List.length xs) (\<lambda>n. xs ! n)" |
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
354 |
by (rule Heap_eqI) (simp add: map_nth execute_simps) |
26170 | 355 |
|
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
356 |
hide_const (open) present get set alloc length update noteq new of_list make len nth upd map_entry swap freeze |
26170 | 357 |
|
26182 | 358 |
|
359 |
subsection {* Code generator setup *} |
|
360 |
||
361 |
subsubsection {* Logical intermediate layer *} |
|
362 |
||
363 |
definition new' where |
|
31205
98370b26c2ce
String.literal replaces message_string, code_numeral replaces (code_)index
haftmann
parents:
31203
diff
changeset
|
364 |
[code del]: "new' = Array.new o Code_Numeral.nat_of" |
37752 | 365 |
|
28562 | 366 |
lemma [code]: |
37752 | 367 |
"Array.new = new' o Code_Numeral.of_nat" |
26182 | 368 |
by (simp add: new'_def o_def) |
369 |
||
370 |
definition make' where |
|
31205
98370b26c2ce
String.literal replaces message_string, code_numeral replaces (code_)index
haftmann
parents:
31203
diff
changeset
|
371 |
[code del]: "make' i f = Array.make (Code_Numeral.nat_of i) (f o Code_Numeral.of_nat)" |
37752 | 372 |
|
28562 | 373 |
lemma [code]: |
37752 | 374 |
"Array.make n f = make' (Code_Numeral.of_nat n) (f o Code_Numeral.nat_of)" |
26182 | 375 |
by (simp add: make'_def o_def) |
376 |
||
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
377 |
definition len' where |
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
378 |
[code del]: "len' a = Array.len a \<guillemotright>= (\<lambda>n. return (Code_Numeral.of_nat n))" |
37752 | 379 |
|
28562 | 380 |
lemma [code]: |
37752 | 381 |
"Array.len a = len' a \<guillemotright>= (\<lambda>i. return (Code_Numeral.nat_of i))" |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
382 |
by (simp add: len'_def) |
26182 | 383 |
|
384 |
definition nth' where |
|
31205
98370b26c2ce
String.literal replaces message_string, code_numeral replaces (code_)index
haftmann
parents:
31203
diff
changeset
|
385 |
[code del]: "nth' a = Array.nth a o Code_Numeral.nat_of" |
37752 | 386 |
|
28562 | 387 |
lemma [code]: |
37752 | 388 |
"Array.nth a n = nth' a (Code_Numeral.of_nat n)" |
26182 | 389 |
by (simp add: nth'_def) |
390 |
||
391 |
definition upd' where |
|
31205
98370b26c2ce
String.literal replaces message_string, code_numeral replaces (code_)index
haftmann
parents:
31203
diff
changeset
|
392 |
[code del]: "upd' a i x = Array.upd (Code_Numeral.nat_of i) x a \<guillemotright> return ()" |
37752 | 393 |
|
28562 | 394 |
lemma [code]: |
37752 | 395 |
"Array.upd i x a = upd' a (Code_Numeral.of_nat i) x \<guillemotright> return a" |
37709 | 396 |
by (simp add: upd'_def upd_return) |
26182 | 397 |
|
37752 | 398 |
lemma [code]: |
37798
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
399 |
"Array.map_entry i f a = do { |
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
400 |
x \<leftarrow> Array.nth a i; |
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
401 |
Array.upd i (f x) a |
37792 | 402 |
}" |
37758 | 403 |
by (rule Heap_eqI) (simp add: bind_def guard_def map_entry_def execute_simps) |
26182 | 404 |
|
37752 | 405 |
lemma [code]: |
37798
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
406 |
"Array.swap i x a = do { |
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
407 |
y \<leftarrow> Array.nth a i; |
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
408 |
Array.upd i x a; |
37752 | 409 |
return y |
37792 | 410 |
}" |
37758 | 411 |
by (rule Heap_eqI) (simp add: bind_def guard_def swap_def execute_simps) |
37752 | 412 |
|
413 |
lemma [code]: |
|
37798
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
414 |
"Array.freeze a = do { |
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
415 |
n \<leftarrow> Array.len a; |
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
416 |
Heap_Monad.fold_map (\<lambda>i. Array.nth a i) [0..<n] |
37792 | 417 |
}" |
37752 | 418 |
proof (rule Heap_eqI) |
419 |
fix h |
|
420 |
have *: "List.map |
|
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
421 |
(\<lambda>x. fst (the (if x < Array.length h a |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
422 |
then Some (Array.get h a ! x, h) else None))) |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
423 |
[0..<Array.length h a] = |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
424 |
List.map (List.nth (Array.get h a)) [0..<Array.length h a]" |
37752 | 425 |
by simp |
37804
0145e59c1f6c
qualified names for (almost) all array operations
haftmann
parents:
37803
diff
changeset
|
426 |
have "execute (Heap_Monad.fold_map (Array.nth a) [0..<Array.length h a]) h = |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
427 |
Some (Array.get h a, h)" |
37756
59caa6180fff
avoid slightly odd "M" suffix; rename mapM to fold_map (fold_map_abort would be more correct, though)
haftmann
parents:
37752
diff
changeset
|
428 |
apply (subst execute_fold_map_unchanged_heap) |
37752 | 429 |
apply (simp_all add: nth_def guard_def *) |
430 |
apply (simp add: length_def map_nth) |
|
431 |
done |
|
37792 | 432 |
then have "execute (do { |
37798
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
433 |
n \<leftarrow> Array.len a; |
37756
59caa6180fff
avoid slightly odd "M" suffix; rename mapM to fold_map (fold_map_abort would be more correct, though)
haftmann
parents:
37752
diff
changeset
|
434 |
Heap_Monad.fold_map (Array.nth a) [0..<n] |
37806
a7679be14442
qualified names for (really) all array operations
haftmann
parents:
37805
diff
changeset
|
435 |
}) h = Some (Array.get h a, h)" |
37787
30dc3abf4a58
theorem collections do not contain default rules any longer
haftmann
parents:
37771
diff
changeset
|
436 |
by (auto intro: execute_bind_eq_SomeI simp add: execute_simps) |
37798
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
437 |
then show "execute (Array.freeze a) h = execute (do { |
0b0570445a2a
proper merge of operation changes and generic do-syntax
haftmann
parents:
37797
diff
changeset
|
438 |
n \<leftarrow> Array.len a; |
37756
59caa6180fff
avoid slightly odd "M" suffix; rename mapM to fold_map (fold_map_abort would be more correct, though)
haftmann
parents:
37752
diff
changeset
|
439 |
Heap_Monad.fold_map (Array.nth a) [0..<n] |
37792 | 440 |
}) h" by (simp add: execute_simps) |
37752 | 441 |
qed |
442 |
||
37831
fa3a2e35c4f1
repaired some implementations of imperative operations
haftmann
parents:
37827
diff
changeset
|
443 |
hide_const (open) new' make' len' nth' upd' |
37752 | 444 |
|
445 |
||
446 |
text {* SML *} |
|
26182 | 447 |
|
448 |
code_type array (SML "_/ array") |
|
449 |
code_const Array (SML "raise/ (Fail/ \"bare Array\")") |
|
26752 | 450 |
code_const Array.new' (SML "(fn/ ()/ =>/ Array.array/ ((_),/ (_)))") |
37831
fa3a2e35c4f1
repaired some implementations of imperative operations
haftmann
parents:
37827
diff
changeset
|
451 |
code_const Array.of_list (SML "(fn/ ()/ =>/ Array.fromList/ _)") |
26752 | 452 |
code_const Array.make' (SML "(fn/ ()/ =>/ Array.tabulate/ ((_),/ (_)))") |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
453 |
code_const Array.len' (SML "(fn/ ()/ =>/ Array.length/ _)") |
26752 | 454 |
code_const Array.nth' (SML "(fn/ ()/ =>/ Array.sub/ ((_),/ (_)))") |
455 |
code_const Array.upd' (SML "(fn/ ()/ =>/ Array.update/ ((_),/ (_),/ (_)))") |
|
39716
d1c12f4ee9ac
treat equality on refs and arrays as primitive operation
haftmann
parents:
39302
diff
changeset
|
456 |
code_const "HOL.equal :: 'a array \<Rightarrow> 'a array \<Rightarrow> bool" (SML infixl 6 "=") |
26182 | 457 |
|
458 |
code_reserved SML Array |
|
459 |
||
460 |
||
37752 | 461 |
text {* OCaml *} |
26182 | 462 |
|
463 |
code_type array (OCaml "_/ array") |
|
464 |
code_const Array (OCaml "failwith/ \"bare Array\"") |
|
32580 | 465 |
code_const Array.new' (OCaml "(fun/ ()/ ->/ Array.make/ (Big'_int.int'_of'_big'_int/ _)/ _)") |
37831
fa3a2e35c4f1
repaired some implementations of imperative operations
haftmann
parents:
37827
diff
changeset
|
466 |
code_const Array.of_list (OCaml "(fun/ ()/ ->/ Array.of'_list/ _)") |
fa3a2e35c4f1
repaired some implementations of imperative operations
haftmann
parents:
37827
diff
changeset
|
467 |
code_const Array.make' (OCaml "(fun/ ()/ ->/ Array.init/ (Big'_int.int'_of'_big'_int/ _)/ |
fa3a2e35c4f1
repaired some implementations of imperative operations
haftmann
parents:
37827
diff
changeset
|
468 |
(fun k'_ ->/ _/ (Big'_int.big'_int'_of'_int/ k'_)))") |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
469 |
code_const Array.len' (OCaml "(fun/ ()/ ->/ Big'_int.big'_int'_of'_int/ (Array.length/ _))") |
32580 | 470 |
code_const Array.nth' (OCaml "(fun/ ()/ ->/ Array.get/ _/ (Big'_int.int'_of'_big'_int/ _))") |
471 |
code_const Array.upd' (OCaml "(fun/ ()/ ->/ Array.set/ _/ (Big'_int.int'_of'_big'_int/ _)/ _)") |
|
39716
d1c12f4ee9ac
treat equality on refs and arrays as primitive operation
haftmann
parents:
39302
diff
changeset
|
472 |
code_const "HOL.equal :: 'a array \<Rightarrow> 'a array \<Rightarrow> bool" (OCaml infixl 4 "=") |
26182 | 473 |
|
474 |
code_reserved OCaml Array |
|
475 |
||
476 |
||
37752 | 477 |
text {* Haskell *} |
26182 | 478 |
|
29793 | 479 |
code_type array (Haskell "Heap.STArray/ Heap.RealWorld/ _") |
26182 | 480 |
code_const Array (Haskell "error/ \"bare Array\"") |
37831
fa3a2e35c4f1
repaired some implementations of imperative operations
haftmann
parents:
37827
diff
changeset
|
481 |
code_const Array.new' (Haskell "Heap.newArray") |
fa3a2e35c4f1
repaired some implementations of imperative operations
haftmann
parents:
37827
diff
changeset
|
482 |
code_const Array.of_list (Haskell "Heap.newListArray") |
fa3a2e35c4f1
repaired some implementations of imperative operations
haftmann
parents:
37827
diff
changeset
|
483 |
code_const Array.make' (Haskell "Heap.newFunArray") |
37719
271ecd4fb9f9
moved "open" operations from Heap.thy to Array.thy and Ref.thy
haftmann
parents:
37716
diff
changeset
|
484 |
code_const Array.len' (Haskell "Heap.lengthArray") |
29793 | 485 |
code_const Array.nth' (Haskell "Heap.readArray") |
486 |
code_const Array.upd' (Haskell "Heap.writeArray") |
|
39716
d1c12f4ee9ac
treat equality on refs and arrays as primitive operation
haftmann
parents:
39302
diff
changeset
|
487 |
code_const "HOL.equal :: 'a array \<Rightarrow> 'a array \<Rightarrow> bool" (Haskell infix 4 "==") |
d1c12f4ee9ac
treat equality on refs and arrays as primitive operation
haftmann
parents:
39302
diff
changeset
|
488 |
code_instance array :: HOL.equal (Haskell -) |
26182 | 489 |
|
37842 | 490 |
|
491 |
text {* Scala *} |
|
492 |
||
37845
b70d7a347964
first roughly working version of Imperative HOL for Scala
haftmann
parents:
37842
diff
changeset
|
493 |
code_type array (Scala "!collection.mutable.ArraySeq[_]") |
37842 | 494 |
code_const Array (Scala "!error(\"bare Array\")") |
38968
e55deaa22fff
do not print object frame around Scala includes -- this is in the responsibility of the user
haftmann
parents:
38771
diff
changeset
|
495 |
code_const Array.new' (Scala "('_: Unit)/ => / Array.alloc((_))((_))") |
e55deaa22fff
do not print object frame around Scala includes -- this is in the responsibility of the user
haftmann
parents:
38771
diff
changeset
|
496 |
code_const Array.make' (Scala "('_: Unit)/ =>/ Array.make((_))((_))") |
e55deaa22fff
do not print object frame around Scala includes -- this is in the responsibility of the user
haftmann
parents:
38771
diff
changeset
|
497 |
code_const Array.len' (Scala "('_: Unit)/ =>/ Array.len((_))") |
e55deaa22fff
do not print object frame around Scala includes -- this is in the responsibility of the user
haftmann
parents:
38771
diff
changeset
|
498 |
code_const Array.nth' (Scala "('_: Unit)/ =>/ Array.nth((_), (_))") |
e55deaa22fff
do not print object frame around Scala includes -- this is in the responsibility of the user
haftmann
parents:
38771
diff
changeset
|
499 |
code_const Array.upd' (Scala "('_: Unit)/ =>/ Array.upd((_), (_), (_))") |
e55deaa22fff
do not print object frame around Scala includes -- this is in the responsibility of the user
haftmann
parents:
38771
diff
changeset
|
500 |
code_const Array.freeze (Scala "('_: Unit)/ =>/ Array.freeze((_))") |
39716
d1c12f4ee9ac
treat equality on refs and arrays as primitive operation
haftmann
parents:
39302
diff
changeset
|
501 |
code_const "HOL.equal :: 'a array \<Rightarrow> 'a array \<Rightarrow> bool" (Scala infixl 5 "==") |
37842 | 502 |
|
26170 | 503 |
end |