src/HOL/NanoJava/State.thy
changeset 11497 0e66e0114d9a
parent 11376 bf98ad1c22c6
child 11499 7a7bb59a05db
--- a/src/HOL/NanoJava/State.thy	Thu Aug 09 19:33:22 2001 +0200
+++ b/src/HOL/NanoJava/State.thy	Thu Aug 09 20:48:57 2001 +0200
@@ -10,8 +10,8 @@
 
 constdefs
 
-  body :: "cname => mname => stmt"
- "body C m \<equiv> bdy (the (method C m))"
+  body :: "imname => stmt"
+ "body \<equiv> \<lambda>(C,m). bdy (the (method C m))"
 
 text {* locations, i.e.\ abstract references to objects *}
 typedecl loc 
@@ -53,8 +53,11 @@
 
 constdefs
 
+  reset_locs     :: "state => state"
+ "reset_locs s \<equiv> s (| locals := empty |)"
+
   init_locs     :: "cname => mname => state => state"
- "init_locs C m s \<equiv> s (| locals:=init_vars (map_of (lcl (the (method C m))))|)"
+ "init_locs C m s \<equiv> s (| locals:=init_vars (map_of (lcl (the (method C m)))) |)"
 
 text {* The first parameter of @{term set_locs} is of type @{typ state} 
         rather than @{typ locals} in order to keep @{typ locals} private.*}