diff -r ff13585fbdab -r d8d0f8f51d69 src/HOL/ex/PER.thy --- a/src/HOL/ex/PER.thy Sat May 27 17:42:00 2006 +0200 +++ b/src/HOL/ex/PER.thy Sat May 27 17:42:02 2006 +0200 @@ -44,9 +44,9 @@ \emph{any} other one. *} -constdefs - domain :: "'a::partial_equiv set" - "domain == {x. x \ x}" +definition + "domain" :: "'a::partial_equiv set" + "domain = {x. x \ x}" lemma domainI [intro]: "x \ x ==> x \ domain" by (unfold domain_def) blast @@ -164,9 +164,9 @@ representation of elements of a quotient type. *} -constdefs +definition eqv_class :: "('a::partial_equiv) => 'a quot" ("\_\") - "\a\ == Abs_quot {x. a \ x}" + "\a\ = Abs_quot {x. a \ x}" theorem quot_rep: "\a. A = \a\" proof (cases A) @@ -231,9 +231,9 @@ subsection {* Picking representing elements *} -constdefs +definition pick :: "'a::partial_equiv quot => 'a" - "pick A == SOME a. A = \a\" + "pick A = (SOME a. A = \a\)" theorem pick_eqv' [intro?, simp]: "a \ domain ==> pick \a\ \ a" proof (unfold pick_def)