src/HOL/NanoJava/State.thy
changeset 42463 f270e3e18be5
parent 35431 8758fe1fc9f8
child 55466 786edc984c98
--- a/src/HOL/NanoJava/State.thy	Fri Apr 22 15:57:43 2011 +0200
+++ b/src/HOL/NanoJava/State.thy	Sat Apr 23 13:00:19 2011 +0200
@@ -17,9 +17,10 @@
   = Null        --{* null reference *}
   | Addr loc    --{* address, i.e. location of object *}
 
-types   fields
+type_synonym fields
         = "(fname \<rightharpoonup> val)"
 
+type_synonym
         obj = "cname \<times> fields"
 
 translations
@@ -30,8 +31,8 @@
  "init_vars m == Option.map (\<lambda>T. Null) o m"
   
 text {* private: *}
-types   heap   = "loc   \<rightharpoonup> obj"
-        locals = "vname \<rightharpoonup> val"  
+type_synonym heap = "loc   \<rightharpoonup> obj"
+type_synonym locals = "vname \<rightharpoonup> val"  
 
 text {* private: *}
 record  state