src/HOL/Equiv_Relations.thy
changeset 45969 562e99c3d316
parent 44890 22f665a2e91c
child 46752 e9e7209eb375
--- a/src/HOL/Equiv_Relations.thy	Sat Dec 24 15:53:10 2011 +0100
+++ b/src/HOL/Equiv_Relations.thy	Sat Dec 24 15:53:10 2011 +0100
@@ -364,7 +364,7 @@
 
 lemma part_equivpI:
   "(\<exists>x. R x x) \<Longrightarrow> symp R \<Longrightarrow> transp R \<Longrightarrow> part_equivp R"
-  by (auto simp add: part_equivp_def mem_def) (auto elim: sympE transpE)
+  by (auto simp add: part_equivp_def) (auto elim: sympE transpE)
 
 lemma part_equivpE:
   assumes "part_equivp R"
@@ -413,7 +413,7 @@
 
 lemma equivpI:
   "reflp R \<Longrightarrow> symp R \<Longrightarrow> transp R \<Longrightarrow> equivp R"
-  by (auto elim: reflpE sympE transpE simp add: equivp_def mem_def)
+  by (auto elim: reflpE sympE transpE simp add: equivp_def)
 
 lemma equivpE:
   assumes "equivp R"