src/HOL/UNITY/SubstAx.thy
changeset 6575 70d758762c50
parent 6536 281d44905cab
child 8041 e3237d8c18d6
--- a/src/HOL/UNITY/SubstAx.thy	Tue May 04 13:32:53 1999 +0200
+++ b/src/HOL/UNITY/SubstAx.thy	Tue May 04 13:47:28 1999 +0200
@@ -13,6 +13,5 @@
 
 defs
    LeadsTo_def
-    "A LeadsTo B == {F. F : (reachable F  Int  A) leadsTo
-	   	            (reachable F  Int  B)}"
+    "A LeadsTo B == {F. F : (reachable F Int A) leadsTo  B}"
 end