src/ZF/UNITY/Mutex.thy
changeset 41779 a68f503805ed
parent 32960 69916a850301
child 42814 5af15f1e2ef6
--- a/src/ZF/UNITY/Mutex.thy	Fri Feb 18 16:36:42 2011 +0100
+++ b/src/ZF/UNITY/Mutex.thy	Fri Feb 18 17:03:30 2011 +0100
@@ -27,11 +27,11 @@
 abbreviation "u == Var([0,1])"
 abbreviation "v == Var([1,0])"
 
-axioms --{** Type declarations  **}
-  p_type:  "type_of(p)=bool & default_val(p)=0"
-  m_type:  "type_of(m)=int  & default_val(m)=#0"
-  n_type:  "type_of(n)=int  & default_val(n)=#0"
-  u_type:  "type_of(u)=bool & default_val(u)=0"
+axiomatization where --{** Type declarations  **}
+  p_type:  "type_of(p)=bool & default_val(p)=0" and
+  m_type:  "type_of(m)=int  & default_val(m)=#0" and
+  n_type:  "type_of(n)=int  & default_val(n)=#0" and
+  u_type:  "type_of(u)=bool & default_val(u)=0" and
   v_type:  "type_of(v)=bool & default_val(v)=0"
 
 definition