src/ZF/UNITY/AllocBase.thy
changeset 67443 3abf6a722518
parent 61798 27f3c10b0b50
child 69593 3dda49e08b9d
--- a/src/ZF/UNITY/AllocBase.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/ZF/UNITY/AllocBase.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -45,11 +45,11 @@
    "all_distinct(l) == all_distinct0(l)=1"
   
 definition  
-  state_of :: "i =>i" \<comment>\<open>coersion from anyting to state\<close>  where
+  state_of :: "i =>i" \<comment> \<open>coersion from anyting to state\<close>  where
    "state_of(s) == if s \<in> state then s else st0"
 
 definition
-  lift :: "i =>(i=>i)" \<comment>\<open>simplifies the expression of programs\<close>  where
+  lift :: "i =>(i=>i)" \<comment> \<open>simplifies the expression of programs\<close>  where
    "lift(x) == %s. s`x"
 
 text\<open>function to show that the set of variables is infinite\<close>