src/HOL/Equiv_Relations.thy
changeset 21749 3f0e86c92ff3
parent 21404 eb85850d3eb7
child 23705 315c638d5856
--- a/src/HOL/Equiv_Relations.thy	Sun Dec 10 15:30:48 2006 +0100
+++ b/src/HOL/Equiv_Relations.thy	Sun Dec 10 15:30:49 2006 +0100
@@ -224,7 +224,7 @@
 text{*Abbreviation for the common case where the relations are identical*}
 abbreviation
   RESPECTS2:: "['a => 'a => 'b, ('a * 'a) set] => bool"
-    (infixr "respects2 " 80) where
+    (infixr "respects2" 80) where
   "f respects2 r == congruent2 r r f"