src/HOL/Algebra/Coset.thy
changeset 30240 5b25fee0362c
parent 29237 e90d9d51106b
child 31727 2621a957d417
equal deleted inserted replaced
30239:179ff9cb160b 30240:5b25fee0362c
   600    shows "equiv (carrier G) (rcong H)"
   600    shows "equiv (carrier G) (rcong H)"
   601 proof -
   601 proof -
   602   interpret group G by fact
   602   interpret group G by fact
   603   show ?thesis
   603   show ?thesis
   604   proof (intro equiv.intro)
   604   proof (intro equiv.intro)
   605     show "refl (carrier G) (rcong H)"
   605     show "refl_on (carrier G) (rcong H)"
   606       by (auto simp add: r_congruent_def refl_def) 
   606       by (auto simp add: r_congruent_def refl_on_def) 
   607   next
   607   next
   608     show "sym (rcong H)"
   608     show "sym (rcong H)"
   609     proof (simp add: r_congruent_def sym_def, clarify)
   609     proof (simp add: r_congruent_def sym_def, clarify)
   610       fix x y
   610       fix x y
   611       assume [simp]: "x \<in> carrier G" "y \<in> carrier G" 
   611       assume [simp]: "x \<in> carrier G" "y \<in> carrier G"