src/HOL/UNITY/Reach.thy
changeset 6535 880f31a62784
parent 6295 351b3c2b0d83
child 10064 1a77667b21ef
--- a/src/HOL/UNITY/Reach.thy	Tue Apr 27 15:39:43 1999 +0200
+++ b/src/HOL/UNITY/Reach.thy	Wed Apr 28 13:36:31 1999 +0200
@@ -6,7 +6,7 @@
 Reachability in Directed Graphs.  From Chandy and Misra, section 6.4.
 *)
 
-Reach = FP + Traces + SubstAx +
+Reach = FP + SubstAx +
 
 types   vertex
         state = "vertex=>bool"