# HG changeset patch # User wenzelm # Date 975611134 -3600 # Node ID ec9fab41b3a08d6995a5cc021387bdf56ebeba3c # Parent 93ca45370c593e673847079016072f8e8e851a9e renamed "equivalence_class" to "class"; diff -r 93ca45370c59 -r ec9fab41b3a0 src/HOL/Library/Quotient.thy --- a/src/HOL/Library/Quotient.thy Thu Nov 30 20:05:10 2000 +0100 +++ b/src/HOL/Library/Quotient.thy Thu Nov 30 20:05:34 2000 +0100 @@ -76,7 +76,7 @@ *} constdefs - equivalence_class :: "'a::equiv => 'a quot" ("\_\") + class :: "'a::equiv => 'a quot" ("\_\") "\a\ == Abs_quot {x. a \ x}" theorem quot_exhaust: "\a. A = \a\" @@ -84,7 +84,7 @@ fix R assume R: "A = Abs_quot R" assume "R \ quot" hence "\a. R = {x. a \ x}" by blast with R have "\a. A = Abs_quot {x. a \ x}" by blast - thus ?thesis by (unfold equivalence_class_def) + thus ?thesis by (unfold class_def) qed lemma quot_cases [cases type: quot]: "(!!a. A = \a\ ==> C) ==> C" @@ -104,7 +104,7 @@ show "a \ b" proof - from eq have "{x. a \ x} = {x. b \ x}" - by (simp only: equivalence_class_def Abs_quot_inject quotI) + by (simp only: class_def Abs_quot_inject quotI) moreover have "a \ a" .. ultimately have "a \ {x. b \ x}" by blast hence "b \ a" by blast @@ -127,7 +127,7 @@ finally show "a \ x" . qed qed - thus ?thesis by (simp only: equivalence_class_def) + thus ?thesis by (simp only: class_def) qed qed