src/HOL/NanoJava/State.thy
changeset 35431 8758fe1fc9f8
parent 35417 47ee18b6ae32
child 42463 f270e3e18be5
--- a/src/HOL/NanoJava/State.thy	Wed Mar 03 00:32:14 2010 +0100
+++ b/src/HOL/NanoJava/State.thy	Wed Mar 03 00:33:02 2010 +0100
@@ -23,9 +23,8 @@
         obj = "cname \<times> fields"
 
 translations
-
-  "fields" \<leftharpoondown> (type)"fname => val option"
-  "obj"    \<leftharpoondown> (type)"cname \<times> fields"
+  (type) "fields" \<leftharpoondown> (type) "fname => val option"
+  (type) "obj"    \<leftharpoondown> (type) "cname \<times> fields"
 
 definition init_vars :: "('a \<rightharpoonup> 'b) => ('a \<rightharpoonup> val)" where
  "init_vars m == Option.map (\<lambda>T. Null) o m"
@@ -40,10 +39,9 @@
           locals :: locals
 
 translations
-
-  "heap"   \<leftharpoondown> (type)"loc   => obj option"
-  "locals" \<leftharpoondown> (type)"vname => val option"
-  "state" \<leftharpoondown> (type)"(|heap :: heap, locals :: locals|)"
+  (type) "heap" \<leftharpoondown> (type) "loc => obj option"
+  (type) "locals" \<leftharpoondown> (type) "vname => val option"
+  (type) "state" \<leftharpoondown> (type) "(|heap :: heap, locals :: locals|)"
 
 definition del_locs :: "state => state" where
  "del_locs s \<equiv> s (| locals := empty |)"