src/ZF/ex/Ramsey.thy
changeset 38 4433428596f9
parent 0 a5a9c433f639
child 753 ec86863e87c8
--- a/src/ZF/ex/Ramsey.thy	Thu Oct 07 10:48:16 1993 +0100
+++ b/src/ZF/ex/Ramsey.thy	Thu Oct 07 11:47:50 1993 +0100
@@ -30,10 +30,10 @@
     "Symmetric(E) == (ALL x y. <x,y>:E --> <y,x>:E)"
 
   Clique_def
-    "Clique(C,V,E) == (C<=V) & (ALL x:C. ALL y:C. ~ x=y --> <x,y>:E)"
+    "Clique(C,V,E) == (C<=V) & (ALL x:C. ALL y:C. x~=y --> <x,y> : E)"
 
   Indept_def
-    "Indept(I,V,E) == (I<=V) & (ALL x:I. ALL y:I. ~ x=y --> ~ <x,y>:E)"
+    "Indept(I,V,E) == (I<=V) & (ALL x:I. ALL y:I. x~=y --> <x,y> ~: E)"
 
   Atleast_def
     "Atleast(n,S) == (EX f. f: inj(n,S))"