src/HOL/Library/Quotient.thy
changeset 21404 eb85850d3eb7
parent 19086 1b3780be6cc2
child 22390 378f34b1e380
--- a/src/HOL/Library/Quotient.thy	Fri Nov 17 02:19:55 2006 +0100
+++ b/src/HOL/Library/Quotient.thy	Fri Nov 17 02:20:03 2006 +0100
@@ -75,7 +75,7 @@
 *}
 
 definition
-  "class" :: "'a::equiv => 'a quot"    ("\<lfloor>_\<rfloor>")
+  "class" :: "'a::equiv => 'a quot"  ("\<lfloor>_\<rfloor>") where
   "\<lfloor>a\<rfloor> = Abs_quot {x. a \<sim> x}"
 
 theorem quot_exhaust: "\<exists>a. A = \<lfloor>a\<rfloor>"
@@ -134,7 +134,7 @@
 subsection {* Picking representing elements *}
 
 definition
-  pick :: "'a::equiv quot => 'a"
+  pick :: "'a::equiv quot => 'a" where
   "pick A = (SOME a. A = \<lfloor>a\<rfloor>)"
 
 theorem pick_equiv [intro]: "pick \<lfloor>a\<rfloor> \<sim> a"