src/ZF/UNITY/AllocImpl.thy
changeset 41779 a68f503805ed
parent 32960 69916a850301
child 46823 57bf0cecb366
--- a/src/ZF/UNITY/AllocImpl.thy	Fri Feb 18 16:36:42 2011 +0100
+++ b/src/ZF/UNITY/AllocImpl.thy	Fri Feb 18 17:03:30 2011 +0100
@@ -16,9 +16,9 @@
   available_tok :: i  (*number of free tokens (T in paper)*)  where
   "available_tok == Var([succ(succ(2))])"
 
-axioms
+axiomatization where
   alloc_type_assumes [simp]:
-  "type_of(NbR) = nat & type_of(available_tok)=nat"
+  "type_of(NbR) = nat & type_of(available_tok)=nat" and
 
   alloc_default_val_assumes [simp]:
   "default_val(NbR)  = 0 & default_val(available_tok)=0"