src/HOL/UNITY/Comp/TimerArray.thy
changeset 16417 9bc16273c2d4
parent 16184 80617b8d33c5
child 18556 dc39832e9280
--- a/src/HOL/UNITY/Comp/TimerArray.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/UNITY/Comp/TimerArray.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
 A trivial example of reasoning about an array of processes
 *)
 
-theory TimerArray = UNITY_Main:
+theory TimerArray imports UNITY_Main begin
 
 types 'a state = "nat * 'a"   (*second component allows new variables*)