diff -r dd58f13a8eb4 -r eb85850d3eb7 src/HOL/Library/Quotient.thy --- 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" ("\_\") + "class" :: "'a::equiv => 'a quot" ("\_\") where "\a\ = Abs_quot {x. a \ x}" theorem quot_exhaust: "\a. A = \a\" @@ -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 = \a\)" theorem pick_equiv [intro]: "pick \a\ \ a"