diff -r 23a8c5ac35f8 -r 69916a850301 src/HOL/Algebra/Coset.thy --- a/src/HOL/Algebra/Coset.thy Sat Oct 17 01:05:59 2009 +0200 +++ b/src/HOL/Algebra/Coset.thy Sat Oct 17 14:43:18 2009 +0200 @@ -609,7 +609,7 @@ proof (simp add: r_congruent_def sym_def, clarify) fix x y assume [simp]: "x \ carrier G" "y \ carrier G" - and "inv x \ y \ H" + and "inv x \ y \ H" hence "inv (inv x \ y) \ H" by (simp add: m_inv_closed) thus "inv y \ x \ H" by (simp add: inv_mult_group) qed @@ -618,10 +618,10 @@ proof (simp add: r_congruent_def trans_def, clarify) fix x y z assume [simp]: "x \ carrier G" "y \ carrier G" "z \ carrier G" - and "inv x \ y \ H" and "inv y \ z \ H" + and "inv x \ y \ H" and "inv y \ z \ H" hence "(inv x \ y) \ (inv y \ z) \ H" by simp hence "inv x \ (y \ inv y) \ z \ H" - by (simp add: m_assoc del: r_inv Units_r_inv) + by (simp add: m_assoc del: r_inv Units_r_inv) thus "inv x \ z \ H" by simp qed qed