diff -r aa157e957655 -r 91b079db7380 Quot/QuotScript.thy --- a/Quot/QuotScript.thy Thu Dec 10 16:56:03 2009 +0100 +++ b/Quot/QuotScript.thy Thu Dec 10 18:28:30 2009 +0100 @@ -31,6 +31,11 @@ shows "equivp E \ (\x y z. E x y \ E y z \ E x z)" by (metis equivp_reflp_symp_transp transp_def) +lemma equivpI: + assumes "reflp R" "symp R" "transp R" + shows "equivp R" +using assms by (simp add: equivp_reflp_symp_transp) + definition "part_equivp E \ (\x. E x x) \ (\x y. E x y = (E x x \ E y y \ (E x = E y)))"