src/HOL/Library/Quotient.thy
changeset 19086 1b3780be6cc2
parent 18730 843da46f89ac
child 21404 eb85850d3eb7
--- a/src/HOL/Library/Quotient.thy	Thu Feb 16 21:11:58 2006 +0100
+++ b/src/HOL/Library/Quotient.thy	Thu Feb 16 21:12:00 2006 +0100
@@ -74,9 +74,9 @@
  representation of elements of a quotient type.
 *}
 
-constdefs
+definition
   "class" :: "'a::equiv => 'a quot"    ("\<lfloor>_\<rfloor>")
-  "\<lfloor>a\<rfloor> == Abs_quot {x. a \<sim> x}"
+  "\<lfloor>a\<rfloor> = Abs_quot {x. a \<sim> x}"
 
 theorem quot_exhaust: "\<exists>a. A = \<lfloor>a\<rfloor>"
 proof (cases A)
@@ -133,9 +133,9 @@
 
 subsection {* Picking representing elements *}
 
-constdefs
+definition
   pick :: "'a::equiv quot => 'a"
-  "pick A == SOME a. A = \<lfloor>a\<rfloor>"
+  "pick A = (SOME a. A = \<lfloor>a\<rfloor>)"
 
 theorem pick_equiv [intro]: "pick \<lfloor>a\<rfloor> \<sim> a"
 proof (unfold pick_def)