src/HOL/UNITY/Constrains.thy
changeset 6575 70d758762c50
parent 6570 a7d7985050a9
child 6705 b2662096ccd0
--- a/src/HOL/UNITY/Constrains.thy	Tue May 04 13:32:53 1999 +0200
+++ b/src/HOL/UNITY/Constrains.thy	Tue May 04 13:47:28 1999 +0200
@@ -36,7 +36,7 @@
 
 defs
   Constrains_def
-    "A Co B == {F. F : (reachable F  Int  A) co (reachable F  Int  B)}"
+    "A Co B == {F. F : (reachable F Int A)  co  B}"
 
   Unless_def
     "A Unless B == (A-B) Co (A Un B)"