src/HOL/Integ/Equiv.thy
changeset 10797 028d22926a41
parent 9392 c8e6529cc082
child 10834 a7897aebbffc
--- a/src/HOL/Integ/Equiv.thy	Fri Jan 05 18:33:47 2001 +0100
+++ b/src/HOL/Integ/Equiv.thy	Fri Jan 05 18:48:18 2001 +0100
@@ -12,7 +12,7 @@
     "equiv A r == refl A r & sym(r) & trans(r)"
 
   quotient :: "['a set, ('a*'a) set] => 'a set set"  (infixl "'/'/" 90) 
-    "A//r == UN x:A. {r^^{x}}"      (*set of equiv classes*)
+    "A//r == UN x:A. {r```{x}}"      (*set of equiv classes*)
 
   congruent  :: "[('a*'a) set, 'a=>'b] => bool"
     "congruent r b  == ALL y z. (y,z):r --> b(y)=b(z)"