src/HOL/Equiv_Relations.thy
changeset 37767 a2b7a20d6ea3
parent 35725 4d7e3cc9c52c
child 40812 ff16e22e8776
--- a/src/HOL/Equiv_Relations.thy	Mon Jul 12 08:58:27 2010 +0200
+++ b/src/HOL/Equiv_Relations.thy	Mon Jul 12 10:48:37 2010 +0200
@@ -93,7 +93,7 @@
 subsection {* Quotients *}
 
 definition quotient :: "'a set \<Rightarrow> ('a \<times> 'a) set \<Rightarrow> 'a set set"  (infixl "'/'/" 90) where
-  [code del]: "A//r = (\<Union>x \<in> A. {r``{x}})"  -- {* set of equiv classes *}
+  "A//r = (\<Union>x \<in> A. {r``{x}})"  -- {* set of equiv classes *}
 
 lemma quotientI: "x \<in> A ==> r``{x} \<in> A//r"
   by (unfold quotient_def) blast