src/HOL/UNITY/Simple/Reachability.thy
changeset 16417 9bc16273c2d4
parent 13806 fd40c9d9076b
child 23767 7272a839ccd9
--- a/src/HOL/UNITY/Simple/Reachability.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/UNITY/Simple/Reachability.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -8,7 +8,7 @@
 From Chandy and Misra, "Parallel Program Design" (1989), sections 6.2 and 11.3
 *)
 
-theory Reachability = Detects + Reach:
+theory Reachability imports Detects Reach begin
 
 types  edge = "(vertex*vertex)"