src/HOL/NanoJava/State.thy
changeset 67443 3abf6a722518
parent 63167 0909deb8059b
child 68451 c34aa23a1fb6
--- a/src/HOL/NanoJava/State.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/NanoJava/State.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -14,8 +14,8 @@
 typedecl loc 
 
 datatype val
-  = Null        \<comment>\<open>null reference\<close>
-  | Addr loc    \<comment>\<open>address, i.e. location of object\<close>
+  = Null        \<comment> \<open>null reference\<close>
+  | Addr loc    \<comment> \<open>address, i.e. location of object\<close>
 
 type_synonym fields
         = "(fname \<rightharpoonup> val)"
@@ -59,7 +59,7 @@
 definition get_local     :: "state => vname => val" ("_<_>" [99,0] 99) where
  "get_local s x  \<equiv> the (locals s x)"
 
-\<comment>\<open>local function:\<close>
+\<comment> \<open>local function:\<close>
 definition get_obj       :: "state => loc => obj" where
  "get_obj s a \<equiv> the (heap s a)"
 
@@ -69,7 +69,7 @@
 definition get_field     :: "state => loc => fname => val" where
  "get_field s a f \<equiv> the (snd (get_obj s a) f)"
 
-\<comment>\<open>local function:\<close>
+\<comment> \<open>local function:\<close>
 definition hupd       :: "loc => obj => state => state"   ("hupd'(_\<mapsto>_')" [10,10] 1000) where
  "hupd a obj s \<equiv> s (| heap   := ((heap   s)(a\<mapsto>obj))|)"