src/HOL/Equiv_Relations.thy
changeset 28229 4f06fae6a55e
parent 26791 3581a9c71909
child 28562 4e74209f113e
--- a/src/HOL/Equiv_Relations.thy	Tue Sep 16 09:21:24 2008 +0200
+++ b/src/HOL/Equiv_Relations.thy	Tue Sep 16 09:21:26 2008 +0200
@@ -93,9 +93,8 @@
 
 subsection {* Quotients *}
 
-constdefs
-  quotient :: "['a set, ('a*'a) set] => 'a set set"  (infixl "'/'/" 90)
-  "A//r == \<Union>x \<in> A. {r``{x}}"  -- {* set of equiv classes *}
+definition quotient :: "'a set \<Rightarrow> ('a \<times> 'a) set \<Rightarrow> 'a set set"  (infixl "'/'/" 90) where
+  [code func del]: "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