src/HOL/UNITY/Comp/Client.thy
changeset 16417 9bc16273c2d4
parent 16184 80617b8d33c5
child 32960 69916a850301
--- a/src/HOL/UNITY/Comp/Client.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/UNITY/Comp/Client.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
 
 header{*Distributed Resource Management System: the Client*}
 
-theory Client = Rename + AllocBase:
+theory Client imports Rename AllocBase begin
 
 types
   tokbag = nat	   --{*tokbags could be multisets...or any ordered type?*}