src/HOL/Algebra/AbelCoset.thy
changeset 62343 24106dc44def
parent 61565 352c73a689da
child 63167 0909deb8059b
equal deleted inserted replaced
62342:1cf129590be8 62343:24106dc44def
   256     fix x
   256     fix x
   257     assume xcarr: "x \<in> carrier G"
   257     assume xcarr: "x \<in> carrier G"
   258     from a_subgroup have Hcarr: "H \<subseteq> carrier G"
   258     from a_subgroup have Hcarr: "H \<subseteq> carrier G"
   259       unfolding subgroup_def by simp
   259       unfolding subgroup_def by simp
   260     from xcarr Hcarr show "(\<Union>h\<in>H. {h \<oplus>\<^bsub>G\<^esub> x}) = (\<Union>h\<in>H. {x \<oplus>\<^bsub>G\<^esub> h})"
   260     from xcarr Hcarr show "(\<Union>h\<in>H. {h \<oplus>\<^bsub>G\<^esub> x}) = (\<Union>h\<in>H. {x \<oplus>\<^bsub>G\<^esub> h})"
   261       using m_comm [simplified] by fast
   261       using m_comm [simplified] by fastforce
   262   qed
   262   qed
   263 qed
   263 qed
   264 
   264 
   265 lemma abelian_subgroupI3:
   265 lemma abelian_subgroupI3:
   266   fixes G (structure)
   266   fixes G (structure)