src/HOL/Algebra/Coset.thy
changeset 40815 6e2d17cc0d1d
parent 39910 10097e0a9dbd
child 41528 276078f01ada
--- a/src/HOL/Algebra/Coset.thy	Mon Nov 29 12:15:14 2010 +0100
+++ b/src/HOL/Algebra/Coset.thy	Mon Nov 29 13:44:54 2010 +0100
@@ -606,7 +606,7 @@
 proof -
   interpret group G by fact
   show ?thesis
-  proof (intro equiv.intro)
+  proof (intro equivI)
     show "refl_on (carrier G) (rcong H)"
       by (auto simp add: r_congruent_def refl_on_def) 
   next