src/HOL/Quotient.thy
changeset 56073 29e308b56d23
parent 55945 e96383acecf9
child 57960 ee1ba4848896
--- a/src/HOL/Quotient.thy	Wed Mar 12 22:57:50 2014 +0100
+++ b/src/HOL/Quotient.thy	Thu Mar 13 07:07:07 2014 +0100
@@ -487,15 +487,7 @@
 
 lemma bex1_bexeq_reg:
   shows "(\<exists>!x\<in>Respects R. P x) \<longrightarrow> (Bex1_rel R (\<lambda>x. P x))"
-  apply (simp add: Ex1_def Bex1_rel_def in_respects)
-  apply clarify
-  apply auto
-  apply (rule bexI)
-  apply assumption
-  apply (simp add: in_respects)
-  apply (simp add: in_respects)
-  apply auto
-  done
+  by (auto simp add: Ex1_def Bex1_rel_def Bex_def Ball_def in_respects)
 
 lemma bex1_bexeq_reg_eqv:
   assumes a: "equivp R"