src/HOL/UNITY/Simple/Channel.thy
changeset 18556 dc39832e9280
parent 16417 9bc16273c2d4
child 35416 d8d7d1b785af
--- a/src/HOL/UNITY/Simple/Channel.thy	Tue Jan 03 14:07:17 2006 +0100
+++ b/src/HOL/UNITY/Simple/Channel.thy	Tue Jan 03 15:43:54 2006 +0100
@@ -8,7 +8,7 @@
 From Misra, "A Logic for Concurrent Programming" (1994), section 13.3
 *)
 
-theory Channel imports UNITY_Main begin
+theory Channel imports "../UNITY_Main" begin
 
 types state = "nat set"