changeset 18556 | dc39832e9280 |
parent 16417 | 9bc16273c2d4 |
child 35416 | d8d7d1b785af |
--- a/src/HOL/UNITY/Comp/TimerArray.thy Tue Jan 03 14:07:17 2006 +0100 +++ b/src/HOL/UNITY/Comp/TimerArray.thy Tue Jan 03 15:43:54 2006 +0100 @@ -6,7 +6,7 @@ A trivial example of reasoning about an array of processes *) -theory TimerArray imports UNITY_Main begin +theory TimerArray imports "../UNITY_Main" begin types 'a state = "nat * 'a" (*second component allows new variables*)