src/ZF/ex/Ramsey.thy
changeset 1155 928a16e02f9f
parent 753 ec86863e87c8
child 1401 0c439768f45c
--- a/src/ZF/ex/Ramsey.thy	Thu Jun 22 12:58:39 1995 +0200
+++ b/src/ZF/ex/Ramsey.thy	Thu Jun 22 17:13:05 1995 +0200
@@ -39,8 +39,8 @@
     "Atleast(n,S) == (EX f. f: inj(n,S))"
 
   Ramsey_def
-    "Ramsey(n,i,j) == ALL V E. Symmetric(E) & Atleast(n,V) -->  \
-\         (EX C. Clique(C,V,E) & Atleast(i,C)) |       \
-\         (EX I. Indept(I,V,E) & Atleast(j,I))"
+    "Ramsey(n,i,j) == ALL V E. Symmetric(E) & Atleast(n,V) -->  
+         (EX C. Clique(C,V,E) & Atleast(i,C)) |       
+         (EX I. Indept(I,V,E) & Atleast(j,I))"
 
 end