src/HOL/UNITY/Comp/AllocBase.thy
changeset 45827 66c68453455c
parent 39246 9e58f0499f57
child 46911 6d2a2f0e904e
--- a/src/HOL/UNITY/Comp/AllocBase.thy	Tue Dec 13 14:04:20 2011 +0100
+++ b/src/HOL/UNITY/Comp/AllocBase.thy	Tue Dec 13 15:18:52 2011 +0100
@@ -7,12 +7,10 @@
 
 theory AllocBase imports "../UNITY_Main" begin
 
-consts
-  NbT      :: nat       (*Number of tokens in system*)
-  Nclients :: nat       (*Number of clients*)
+consts Nclients :: nat  (*Number of clients*)
 
-axioms
-  NbT_pos:  "0 < NbT"
+axiomatization NbT :: nat  (*Number of tokens in system*)
+  where NbT_pos: "0 < NbT"
 
 (*This function merely sums the elements of a list*)
 primrec tokens :: "nat list => nat" where