src/HOL/Algebra/Sylow.thy
changeset 69597 ff784d5a5bfb
parent 69272 15e9ed5b28fb
child 76987 4c275405faae
equal deleted inserted replaced
69596:c8a2755bf220 69597:ff784d5a5bfb
   202 end
   202 end
   203 
   203 
   204 
   204 
   205 subsection \<open>Equal Cardinalities of \<open>M\<close> and the Set of Cosets\<close>
   205 subsection \<open>Equal Cardinalities of \<open>M\<close> and the Set of Cosets\<close>
   206 
   206 
   207 text \<open>Injections between @{term M} and @{term "rcosets\<^bsub>G\<^esub> H"} show that
   207 text \<open>Injections between \<^term>\<open>M\<close> and \<^term>\<open>rcosets\<^bsub>G\<^esub> H\<close> show that
   208  their cardinalities are equal.\<close>
   208  their cardinalities are equal.\<close>
   209 
   209 
   210 lemma ElemClassEquiv: "\<lbrakk>equiv A r; C \<in> A // r\<rbrakk> \<Longrightarrow> \<forall>x \<in> C. \<forall>y \<in> C. (x, y) \<in> r"
   210 lemma ElemClassEquiv: "\<lbrakk>equiv A r; C \<in> A // r\<rbrakk> \<Longrightarrow> \<forall>x \<in> C. \<forall>y \<in> C. (x, y) \<in> r"
   211   unfolding equiv_def quotient_def sym_def trans_def by blast
   211   unfolding equiv_def quotient_def sym_def trans_def by blast
   212 
   212 
   337   show ?thesis
   337   show ?thesis
   338     using H_is_subgroup card_H_eq by blast
   338     using H_is_subgroup card_H_eq by blast
   339 qed
   339 qed
   340 
   340 
   341 text \<open>Needed because the locale's automatic definition refers to
   341 text \<open>Needed because the locale's automatic definition refers to
   342   @{term "semigroup G"} and @{term "group_axioms G"} rather than
   342   \<^term>\<open>semigroup G\<close> and \<^term>\<open>group_axioms G\<close> rather than
   343   simply to @{term "group G"}.\<close>
   343   simply to \<^term>\<open>group G\<close>.\<close>
   344 lemma sylow_eq: "sylow G p a m \<longleftrightarrow> group G \<and> sylow_axioms G p a m"
   344 lemma sylow_eq: "sylow G p a m \<longleftrightarrow> group G \<and> sylow_axioms G p a m"
   345   by (simp add: sylow_def group_def)
   345   by (simp add: sylow_def group_def)
   346 
   346 
   347 
   347 
   348 subsection \<open>Sylow's Theorem\<close>
   348 subsection \<open>Sylow's Theorem\<close>