author | nipkow |
Fri, 26 Nov 1999 08:46:59 +0100 | |
changeset 8034 | 6fc37b5c5e98 |
parent 8011 | d14c4e9e9c8e |
child 8038 | a13c3b80d3d4 |
permissions | -rw-r--r-- |
8011 | 1 |
(* Title: HOL/MicroJava/JVM/Store.thy |
2 |
ID: $Id$ |
|
3 |
Author: Cornelia Pusch |
|
4 |
Copyright 1999 Technische Universitaet Muenchen |
|
5 |
||
6 |
The store. |
|
7 |
||
8 |
The JVM builds on many notions already defined in Java. |
|
9 |
Conform provides notions for the type safety proof of the Bytecode Verifier. |
|
10 |
*) |
|
11 |
||
12 |
Store = Conform + |
|
13 |
||
14 |
syntax |
|
8034
6fc37b5c5e98
Various little changes like cmethd -> method and cfield -> field.
nipkow
parents:
8011
diff
changeset
|
15 |
map_apply :: "['a \\<leadsto> 'b,'a] \\<Rightarrow> 'b" ("_ !! _") |
8011 | 16 |
translations |
8034
6fc37b5c5e98
Various little changes like cmethd -> method and cfield -> field.
nipkow
parents:
8011
diff
changeset
|
17 |
"t !! x" == "the (t x)" |
8011 | 18 |
|
19 |
constdefs |
|
20 |
newref :: "('a \\<leadsto> 'b) \\<Rightarrow> 'a" |
|
21 |
"newref s \\<equiv> \\<epsilon>v. s v = None" |
|
22 |
||
23 |
end |