src/HOL/Algebra/Coset.thy
author paulson
Fri, 14 May 2004 16:50:33 +0200
changeset 14747 2eaff69d3d10
parent 14706 71590b7733b7
child 14761 28b5eb4a867f
permissions -rw-r--r--
removal of locale coset
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
14706
71590b7733b7 tuned document;
wenzelm
parents: 14666
diff changeset
     1
(*  Title:      HOL/Algebra/Coset.thy
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
     2
    ID:         $Id$
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
     3
    Author:     Florian Kammueller, with new proofs by L C Paulson
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
     4
*)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
     5
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
     6
header{*Cosets and Quotient Groups*}
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
     7
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
     8
theory Coset = Group + Exponent:
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
     9
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
    10
declare (in group) l_inv [simp] and r_inv [simp]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    11
14651
02b8f3bcf7fe improved notation;
wenzelm
parents: 14530
diff changeset
    12
constdefs (structure G)
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    13
  r_coset    :: "[_, 'a set, 'a] => 'a set"    (infixl "#>\<index>" 60)
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    14
  "H #> a == (% x. x \<otimes> a) ` H"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    15
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    16
  l_coset    :: "[_, 'a, 'a set] => 'a set"    (infixl "<#\<index>" 60)
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    17
  "a <# H == (% x. a \<otimes> x) ` H"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    18
14651
02b8f3bcf7fe improved notation;
wenzelm
parents: 14530
diff changeset
    19
  rcosets  :: "[_, 'a set] => ('a set)set"
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
    20
  "rcosets G H == r_coset G H ` (carrier G)"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    21
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    22
  set_mult  :: "[_, 'a set ,'a set] => 'a set" (infixl "<#>\<index>" 60)
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    23
  "H <#> K == (%(x,y). x \<otimes> y) ` (H \<times> K)"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    24
14651
02b8f3bcf7fe improved notation;
wenzelm
parents: 14530
diff changeset
    25
  set_inv   :: "[_,'a set] => 'a set"
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
    26
  "set_inv G H == m_inv G ` H"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    27
14651
02b8f3bcf7fe improved notation;
wenzelm
parents: 14530
diff changeset
    28
  normal     :: "['a set, _] => bool"       (infixl "<|" 60)
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
    29
  "normal H G == subgroup H G &
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    30
                  (\<forall>x \<in> carrier G. r_coset G H x = l_coset G x H)"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    31
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    32
syntax (xsymbols)
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    33
  normal :: "['a set, ('a,'b) monoid_scheme] => bool"  (infixl "\<lhd>" 60)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    34
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    35
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    36
subsection {*Lemmas Using Locale Constants*}
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    37
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    38
lemma (in group) r_coset_eq: "H #> a = {b . \<exists>h\<in>H. h \<otimes> a = b}"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    39
by (auto simp add: r_coset_def)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    40
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    41
lemma (in group) l_coset_eq: "a <# H = {b . \<exists>h\<in>H. a \<otimes> h = b}"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    42
by (auto simp add: l_coset_def)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    43
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    44
lemma (in group) setrcos_eq: "rcosets G H = {C . \<exists>a\<in>carrier G. C = H #> a}"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    45
by (auto simp add: rcosets_def)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    46
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    47
lemma (in group) set_mult_eq: "H <#> K = {c . \<exists>h\<in>H. \<exists>k\<in>K. c = h \<otimes> k}"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    48
by (simp add: set_mult_def image_def)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    49
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    50
lemma (in group) coset_mult_assoc:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    51
     "[| M \<subseteq> carrier G; g \<in> carrier G; h \<in> carrier G |]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    52
      ==> (M #> g) #> h = M #> (g \<otimes> h)"
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    53
by (force simp add: r_coset_def m_assoc)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    54
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    55
lemma (in group) coset_mult_one [simp]: "M \<subseteq> carrier G ==> M #> \<one> = M"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    56
by (force simp add: r_coset_def)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    57
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    58
lemma (in group) coset_mult_inv1:
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
    59
     "[| M #> (x \<otimes> (inv y)) = M;  x \<in> carrier G ; y \<in> carrier G;
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    60
         M \<subseteq> carrier G |] ==> M #> x = M #> y"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    61
apply (erule subst [of concl: "%z. M #> x = z #> y"])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    62
apply (simp add: coset_mult_assoc m_assoc)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    63
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    64
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    65
lemma (in group) coset_mult_inv2:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    66
     "[| M #> x = M #> y;  x \<in> carrier G;  y \<in> carrier G;  M \<subseteq> carrier G |]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    67
      ==> M #> (x \<otimes> (inv y)) = M "
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    68
apply (simp add: coset_mult_assoc [symmetric])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    69
apply (simp add: coset_mult_assoc)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    70
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    71
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    72
lemma (in group) coset_join1:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    73
     "[| H #> x = H;  x \<in> carrier G;  subgroup H G |] ==> x \<in> H"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    74
apply (erule subst)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    75
apply (simp add: r_coset_eq)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    76
apply (blast intro: l_one subgroup.one_closed)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    77
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    78
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    79
lemma (in group) solve_equation:
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    80
    "\<lbrakk>subgroup H G; x \<in> H; y \<in> H\<rbrakk> \<Longrightarrow> \<exists>h\<in>H. h \<otimes> x = y"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    81
apply (rule bexI [of _ "y \<otimes> (inv x)"])
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
    82
apply (auto simp add: subgroup.m_closed subgroup.m_inv_closed m_assoc
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    83
                      subgroup.subset [THEN subsetD])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    84
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    85
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    86
lemma (in group) coset_join2:
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    87
     "[| x \<in> carrier G;  subgroup H G;  x\<in>H |] ==> H #> x = H"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    88
by (force simp add: subgroup.m_closed r_coset_eq solve_equation)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    89
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    90
lemma (in group) r_coset_subset_G:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    91
     "[| H \<subseteq> carrier G; x \<in> carrier G |] ==> H #> x \<subseteq> carrier G"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    92
by (auto simp add: r_coset_def)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    93
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    94
lemma (in group) rcosI:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    95
     "[| h \<in> H; H \<subseteq> carrier G; x \<in> carrier G|] ==> h \<otimes> x \<in> H #> x"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    96
by (auto simp add: r_coset_def)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
    97
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    98
lemma (in group) setrcosI:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
    99
     "[| H \<subseteq> carrier G; x \<in> carrier G |] ==> H #> x \<in> rcosets G H"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   100
by (auto simp add: setrcos_eq)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   101
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   102
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   103
text{*Really needed?*}
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   104
lemma (in group) transpose_inv:
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   105
     "[| x \<otimes> y = z;  x \<in> carrier G;  y \<in> carrier G;  z \<in> carrier G |]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   106
      ==> (inv x) \<otimes> z = y"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   107
by (force simp add: m_assoc [symmetric])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   108
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   109
lemma (in group) repr_independence:
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   110
     "[| y \<in> H #> x;  x \<in> carrier G; subgroup H G |] ==> H #> x = H #> y"
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   111
by (auto simp add: r_coset_eq m_assoc [symmetric]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   112
                   subgroup.subset [THEN subsetD]
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   113
                   subgroup.m_closed solve_equation)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   114
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   115
lemma (in group) rcos_self: "[| x \<in> carrier G; subgroup H G |] ==> x \<in> H #> x"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   116
apply (simp add: r_coset_eq)
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   117
apply (blast intro: l_one subgroup.subset [THEN subsetD]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   118
                    subgroup.one_closed)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   119
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   120
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   121
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   122
subsection {* Normal subgroups *}
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   123
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   124
lemma normal_imp_subgroup: "H <| G ==> subgroup H G"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   125
by (simp add: normal_def)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   126
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   127
lemma (in group) normal_inv_op_closed1:
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   128
     "\<lbrakk>H \<lhd> G; x \<in> carrier G; h \<in> H\<rbrakk> \<Longrightarrow> (inv x) \<otimes> h \<otimes> x \<in> H"
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   129
apply (auto simp add: l_coset_def r_coset_def normal_def)
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   130
apply (drule bspec, assumption)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   131
apply (drule equalityD1 [THEN subsetD], blast, clarify)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   132
apply (simp add: m_assoc subgroup.subset [THEN subsetD])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   133
apply (simp add: m_assoc [symmetric] subgroup.subset [THEN subsetD])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   134
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   135
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   136
lemma (in group) normal_inv_op_closed2:
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   137
     "\<lbrakk>H \<lhd> G; x \<in> carrier G; h \<in> H\<rbrakk> \<Longrightarrow> x \<otimes> h \<otimes> (inv x) \<in> H"
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   138
apply (drule normal_inv_op_closed1 [of H "(inv x)"])
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   139
apply auto
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   140
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   141
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   142
text{*Alternative characterization of normal subgroups*}
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   143
lemma (in group) normal_inv_iff:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   144
     "(N \<lhd> G) = 
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   145
      (subgroup N G & (\<forall>x \<in> carrier G. \<forall>h \<in> N. x \<otimes> h \<otimes> (inv x) \<in> N))"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   146
      (is "_ = ?rhs")
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   147
proof
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   148
  assume N: "N \<lhd> G"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   149
  show ?rhs
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   150
    by (blast intro: N normal_imp_subgroup normal_inv_op_closed2) 
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   151
next
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   152
  assume ?rhs
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   153
  hence sg: "subgroup N G" 
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   154
    and closed: "!!x. x\<in>carrier G ==> \<forall>h\<in>N. x \<otimes> h \<otimes> inv x \<in> N" by auto
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   155
  hence sb: "N \<subseteq> carrier G" by (simp add: subgroup.subset) 
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   156
  show "N \<lhd> G"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   157
  proof (simp add: sg normal_def l_coset_def r_coset_def, clarify)
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   158
    fix x
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   159
    assume x: "x \<in> carrier G"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   160
    show "(\<lambda>n. n \<otimes> x) ` N = op \<otimes> x ` N"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   161
    proof
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   162
      show "(\<lambda>n. n \<otimes> x) ` N \<subseteq> op \<otimes> x ` N"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   163
      proof clarify
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   164
        fix n
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   165
        assume n: "n \<in> N" 
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   166
        show "n \<otimes> x \<in> op \<otimes> x ` N"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   167
        proof 
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   168
          show "n \<otimes> x = x \<otimes> (inv x \<otimes> n \<otimes> x)"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   169
            by (simp add: x n m_assoc [symmetric] sb [THEN subsetD])
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   170
          with closed [of "inv x"]
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   171
          show "inv x \<otimes> n \<otimes> x \<in> N" by (simp add: x n)
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   172
        qed
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   173
      qed
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   174
    next
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   175
      show "op \<otimes> x ` N \<subseteq> (\<lambda>n. n \<otimes> x) ` N" 
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   176
      proof clarify
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   177
        fix n
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   178
        assume n: "n \<in> N" 
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   179
        show "x \<otimes> n \<in> (\<lambda>n. n \<otimes> x) ` N"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   180
        proof 
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   181
          show "x \<otimes> n = (x \<otimes> n \<otimes> inv x) \<otimes> x"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   182
            by (simp add: x n m_assoc sb [THEN subsetD])
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   183
          show "x \<otimes> n \<otimes> inv x \<in> N" by (simp add: x n closed)
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   184
        qed
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   185
      qed
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   186
    qed
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   187
  qed
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   188
qed
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   189
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   190
lemma (in group) lcos_m_assoc:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   191
     "[| M \<subseteq> carrier G; g \<in> carrier G; h \<in> carrier G |]
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   192
      ==> g <# (h <# M) = (g \<otimes> h) <# M"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   193
by (force simp add: l_coset_def m_assoc)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   194
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   195
lemma (in group) lcos_mult_one: "M \<subseteq> carrier G ==> \<one> <# M = M"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   196
by (force simp add: l_coset_def)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   197
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   198
lemma (in group) l_coset_subset_G:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   199
     "[| H \<subseteq> carrier G; x \<in> carrier G |] ==> x <# H \<subseteq> carrier G"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   200
by (auto simp add: l_coset_def subsetD)
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   201
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   202
lemma (in group) l_coset_swap:
14530
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   203
     "[| y \<in> x <# H;  x \<in> carrier G;  subgroup H G |] ==> x \<in> y <# H"
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   204
proof (simp add: l_coset_eq)
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   205
  assume "\<exists>h\<in>H. x \<otimes> h = y"
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   206
    and x: "x \<in> carrier G"
14530
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   207
    and sb: "subgroup H G"
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   208
  then obtain h' where h': "h' \<in> H & x \<otimes> h' = y" by blast
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   209
  show "\<exists>h\<in>H. y \<otimes> h = x"
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   210
  proof
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   211
    show "y \<otimes> inv h' = x" using h' x sb
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   212
      by (auto simp add: m_assoc subgroup.subset [THEN subsetD])
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   213
    show "inv h' \<in> H" using h' sb
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   214
      by (auto simp add: subgroup.subset [THEN subsetD] subgroup.m_inv_closed)
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   215
  qed
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   216
qed
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   217
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   218
lemma (in group) l_coset_carrier:
14530
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   219
     "[| y \<in> x <# H;  x \<in> carrier G;  subgroup H G |] ==> y \<in> carrier G"
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   220
by (auto simp add: l_coset_def m_assoc
14530
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   221
                   subgroup.subset [THEN subsetD] subgroup.m_closed)
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   222
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   223
lemma (in group) l_repr_imp_subset:
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   224
  assumes y: "y \<in> x <# H" and x: "x \<in> carrier G" and sb: "subgroup H G"
14530
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   225
  shows "y <# H \<subseteq> x <# H"
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   226
proof -
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   227
  from y
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   228
  obtain h' where "h' \<in> H" "x \<otimes> h' = y" by (auto simp add: l_coset_def)
14530
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   229
  thus ?thesis using x sb
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   230
    by (auto simp add: l_coset_def m_assoc
14530
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   231
                       subgroup.subset [THEN subsetD] subgroup.m_closed)
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   232
qed
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   233
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   234
lemma (in group) l_repr_independence:
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   235
  assumes y: "y \<in> x <# H" and x: "x \<in> carrier G" and sb: "subgroup H G"
14530
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   236
  shows "x <# H = y <# H"
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   237
proof
14530
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   238
  show "x <# H \<subseteq> y <# H"
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   239
    by (rule l_repr_imp_subset,
14530
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   240
        (blast intro: l_coset_swap l_coset_carrier y x sb)+)
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   241
  show "y <# H \<subseteq> x <# H" by (rule l_repr_imp_subset [OF y x sb])
14530
e94fd774ecf5 some (much longer) structured proofs
paulson
parents: 14254
diff changeset
   242
qed
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   243
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   244
lemma (in group) setmult_subset_G:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   245
     "[| H \<subseteq> carrier G; K \<subseteq> carrier G |] ==> H <#> K \<subseteq> carrier G"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   246
by (auto simp add: set_mult_eq subsetD)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   247
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   248
lemma (in group) subgroup_mult_id: "subgroup H G ==> H <#> H = H"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   249
apply (auto simp add: subgroup.m_closed set_mult_eq Sigma_def image_def)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   250
apply (rule_tac x = x in bexI)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   251
apply (rule bexI [of _ "\<one>"])
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   252
apply (auto simp add: subgroup.m_closed subgroup.one_closed
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   253
                      r_one subgroup.subset [THEN subsetD])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   254
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   255
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   256
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   257
subsubsection {* Set of inverses of an @{text r_coset}. *}
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   258
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   259
lemma (in group) rcos_inv:
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   260
  assumes normalHG: "H <| G"
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   261
      and x:     "x \<in> carrier G"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   262
  shows "set_inv G (H #> x) = H #> (inv x)"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   263
proof -
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   264
  have H_subset: "H \<subseteq> carrier G"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   265
    by (rule subgroup.subset [OF normal_imp_subgroup, OF normalHG])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   266
  show ?thesis
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   267
  proof (auto simp add: r_coset_eq image_def set_inv_def)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   268
    fix h
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   269
    assume "h \<in> H"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   270
      hence "((inv x) \<otimes> (inv h) \<otimes> x) \<otimes> inv x = inv (h \<otimes> x)"
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   271
        by (simp add: x m_assoc inv_mult_group H_subset [THEN subsetD])
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   272
      thus "\<exists>j\<in>H. j \<otimes> inv x = inv (h \<otimes> x)"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   273
       using prems
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   274
        by (blast intro: normal_inv_op_closed1 normal_imp_subgroup
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   275
                         subgroup.m_inv_closed)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   276
  next
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   277
    fix h
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   278
    assume "h \<in> H"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   279
      hence eq: "(x \<otimes> (inv h) \<otimes> (inv x)) \<otimes> x = x \<otimes> inv h"
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   280
        by (simp add: x m_assoc H_subset [THEN subsetD])
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   281
      hence "(\<exists>j\<in>H. j \<otimes> x = inv  (h \<otimes> (inv x))) \<and> h \<otimes> inv x = inv (inv (h \<otimes> (inv x)))"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   282
       using prems
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   283
        by (simp add: m_assoc inv_mult_group H_subset [THEN subsetD],
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   284
            blast intro: eq normal_inv_op_closed2 normal_imp_subgroup
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   285
                         subgroup.m_inv_closed)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   286
      thus "\<exists>y. (\<exists>h\<in>H. h \<otimes> x = y) \<and> h \<otimes> inv x = inv y" ..
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   287
  qed
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   288
qed
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   289
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   290
lemma (in group) rcos_inv2:
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   291
     "[| H <| G; K \<in> rcosets G H; x \<in> K |] ==> set_inv G K = H #> (inv x)"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   292
apply (simp add: setrcos_eq, clarify)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   293
apply (subgoal_tac "x : carrier G")
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   294
 prefer 2
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   295
 apply (blast dest: r_coset_subset_G subgroup.subset normal_imp_subgroup)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   296
apply (drule repr_independence)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   297
  apply assumption
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   298
 apply (erule normal_imp_subgroup)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   299
apply (simp add: rcos_inv)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   300
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   301
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   302
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   303
subsubsection {* Some rules for @{text "<#>"} with @{text "#>"} or @{text "<#"}. *}
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   304
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   305
lemma (in group) setmult_rcos_assoc:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   306
     "[| H \<subseteq> carrier G; K \<subseteq> carrier G; x \<in> carrier G |]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   307
      ==> H <#> (K #> x) = (H <#> K) #> x"
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   308
apply (auto simp add: r_coset_def set_mult_def)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   309
apply (force simp add: m_assoc)+
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   310
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   311
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   312
lemma (in group) rcos_assoc_lcos:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   313
     "[| H \<subseteq> carrier G; K \<subseteq> carrier G; x \<in> carrier G |]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   314
      ==> (H #> x) <#> K = H <#> (x <# K)"
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   315
apply (auto simp add: r_coset_def l_coset_def set_mult_def Sigma_def image_def)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   316
apply (force intro!: exI bexI simp add: m_assoc)+
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   317
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   318
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   319
lemma (in group) rcos_mult_step1:
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   320
     "[| H <| G; x \<in> carrier G; y \<in> carrier G |]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   321
      ==> (H #> x) <#> (H #> y) = (H <#> (x <# H)) #> y"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   322
by (simp add: setmult_rcos_assoc normal_imp_subgroup [THEN subgroup.subset]
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   323
              r_coset_subset_G l_coset_subset_G rcos_assoc_lcos)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   324
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   325
lemma (in group) rcos_mult_step2:
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   326
     "[| H <| G; x \<in> carrier G; y \<in> carrier G |]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   327
      ==> (H <#> (x <# H)) #> y = (H <#> (H #> x)) #> y"
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   328
by (simp add: normal_def)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   329
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   330
lemma (in group) rcos_mult_step3:
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   331
     "[| H <| G; x \<in> carrier G; y \<in> carrier G |]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   332
      ==> (H <#> (H #> x)) #> y = H #> (x \<otimes> y)"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   333
by (simp add: setmult_rcos_assoc r_coset_subset_G coset_mult_assoc
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   334
              setmult_subset_G  subgroup_mult_id
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   335
              subgroup.subset normal_imp_subgroup)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   336
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   337
lemma (in group) rcos_sum:
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   338
     "[| H <| G; x \<in> carrier G; y \<in> carrier G |]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   339
      ==> (H #> x) <#> (H #> y) = H #> (x \<otimes> y)"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   340
by (simp add: rcos_mult_step1 rcos_mult_step2 rcos_mult_step3)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   341
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   342
lemma (in group) setrcos_mult_eq: "[|H <| G; M \<in> rcosets G H|] ==> H <#> M = M"
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   343
  -- {* generalizes @{text subgroup_mult_id} *}
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   344
  by (auto simp add: setrcos_eq normal_imp_subgroup subgroup.subset
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   345
    setmult_rcos_assoc subgroup_mult_id)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   346
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   347
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   348
subsection {*Lemmas Leading to Lagrange's Theorem *}
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   349
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   350
lemma (in group) setrcos_part_G: "subgroup H G ==> \<Union>rcosets G H = carrier G"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   351
apply (rule equalityI)
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   352
apply (force simp add: subgroup.subset [THEN subsetD]
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   353
                       setrcos_eq r_coset_def)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   354
apply (auto simp add: setrcos_eq subgroup.subset rcos_self)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   355
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   356
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   357
lemma (in group) cosets_finite:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   358
     "[| c \<in> rcosets G H;  H \<subseteq> carrier G;  finite (carrier G) |] ==> finite c"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   359
apply (auto simp add: setrcos_eq)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   360
apply (simp (no_asm_simp) add: r_coset_subset_G [THEN finite_subset])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   361
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   362
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   363
text{*The next two lemmas support the proof of @{text card_cosets_equal}.*}
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   364
lemma (in group) inj_on_f:
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   365
    "[|H \<subseteq> carrier G;  a \<in> carrier G|] ==> inj_on (\<lambda>y. y \<otimes> inv a) (H #> a)"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   366
apply (rule inj_onI)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   367
apply (subgoal_tac "x \<in> carrier G & y \<in> carrier G")
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   368
 prefer 2 apply (blast intro: r_coset_subset_G [THEN subsetD])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   369
apply (simp add: subsetD)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   370
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   371
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   372
lemma (in group) inj_on_g:
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   373
    "[|H \<subseteq> carrier G;  a \<in> carrier G|] ==> inj_on (\<lambda>y. y \<otimes> a) H"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   374
by (force simp add: inj_on_def subsetD)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   375
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   376
lemma (in group) card_cosets_equal:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   377
     "[| c \<in> rcosets G H;  H \<subseteq> carrier G; finite(carrier G) |]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   378
      ==> card c = card H"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   379
apply (auto simp add: setrcos_eq)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   380
apply (rule card_bij_eq)
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   381
     apply (rule inj_on_f, assumption+)
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   382
    apply (force simp add: m_assoc subsetD r_coset_def)
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   383
   apply (rule inj_on_g, assumption+)
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   384
  apply (force simp add: m_assoc subsetD r_coset_def)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   385
 txt{*The sets @{term "H #> a"} and @{term "H"} are finite.*}
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   386
 apply (simp add: r_coset_subset_G [THEN finite_subset])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   387
apply (blast intro: finite_subset)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   388
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   389
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   390
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   391
subsection{*Two distinct right cosets are disjoint*}
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   392
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   393
lemma (in group) rcos_equation:
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   394
     "[|subgroup H G;  a \<in> carrier G;  b \<in> carrier G;  ha \<otimes> a = h \<otimes> b;
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   395
        h \<in> H;  ha \<in> H;  hb \<in> H|]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   396
      ==> \<exists>h\<in>H. h \<otimes> b = hb \<otimes> a"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   397
apply (rule bexI [of _"hb \<otimes> ((inv ha) \<otimes> h)"])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   398
apply (simp  add: m_assoc transpose_inv subgroup.subset [THEN subsetD])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   399
apply (simp add: subgroup.m_closed subgroup.m_inv_closed)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   400
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   401
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   402
lemma (in group) rcos_disjoint:
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   403
     "[|subgroup H G; a \<in> rcosets G H; b \<in> rcosets G H; a\<noteq>b|] ==> a \<inter> b = {}"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   404
apply (simp add: setrcos_eq r_coset_eq)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   405
apply (blast intro: rcos_equation sym)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   406
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   407
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   408
lemma (in group) setrcos_subset_PowG:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   409
     "subgroup H G  ==> rcosets G H \<subseteq> Pow(carrier G)"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   410
apply (simp add: setrcos_eq)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   411
apply (blast dest: r_coset_subset_G subgroup.subset)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   412
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   413
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   414
subsection {*Quotient Groups: Factorization of a Group*}
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   415
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   416
constdefs
13936
d3671b878828 Greatly extended CRing. Added Module.
ballarin
parents: 13889
diff changeset
   417
  FactGroup :: "[('a,'b) monoid_scheme, 'a set] => ('a set) monoid"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   418
     (infixl "Mod" 60)
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   419
    --{*Actually defined for groups rather than monoids*}
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   420
  "FactGroup G H ==
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   421
    (| carrier = rcosets G H,
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   422
       mult = (%X: rcosets G H. %Y: rcosets G H. set_mult G X Y),
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   423
       one = H |)"
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   424
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   425
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   426
lemma (in group) setmult_closed:
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   427
     "[| H <| G; K1 \<in> rcosets G H; K2 \<in> rcosets G H |]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   428
      ==> K1 <#> K2 \<in> rcosets G H"
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   429
by (auto simp add: normal_imp_subgroup [THEN subgroup.subset]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   430
                   rcos_sum setrcos_eq)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   431
13889
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   432
lemma (in group) setinv_closed:
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   433
     "[| H <| G; K \<in> rcosets G H |] ==> set_inv G K \<in> rcosets G H"
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   434
by (auto simp add: normal_imp_subgroup
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   435
                   subgroup.subset rcos_inv
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   436
                   setrcos_eq)
13889
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   437
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   438
(*
13889
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   439
The old version is no longer valid: "group G" has to be an explicit premise.
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   440
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   441
lemma setinv_closed:
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   442
     "[| H <| G; K \<in> rcosets G H |] ==> set_inv G K \<in> rcosets G H"
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   443
by (auto simp add:  normal_imp_subgroup
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   444
                   subgroup.subset coset.rcos_inv coset.setrcos_eq)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   445
*)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   446
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   447
lemma (in group) setrcos_assoc:
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   448
     "[|H <| G; M1 \<in> rcosets G H; M2 \<in> rcosets G H; M3 \<in> rcosets G H|]
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   449
      ==> M1 <#> M2 <#> M3 = M1 <#> (M2 <#> M3)"
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   450
by (auto simp add: setrcos_eq rcos_sum normal_imp_subgroup
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   451
                   subgroup.subset m_assoc)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   452
13889
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   453
lemma (in group) subgroup_in_rcosets:
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   454
  "subgroup H G ==> H \<in> rcosets G H"
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   455
proof -
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   456
  assume sub: "subgroup H G"
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   457
  have "r_coset G H \<one> = H"
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   458
    by (rule coset_join2)
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   459
       (auto intro: sub subgroup.one_closed)
13889
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   460
  then show ?thesis
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   461
    by (auto simp add: setrcos_eq)
13889
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   462
qed
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   463
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   464
(*
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   465
lemma subgroup_in_rcosets:
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   466
  "subgroup H G ==> H \<in> rcosets G H"
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   467
apply (frule subgroup_imp_coset)
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   468
apply (frule subgroup_imp_group)
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   469
apply (simp add: coset.setrcos_eq)
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   470
apply (blast del: equalityI
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   471
             intro!: group.subgroup.one_closed group.one_closed
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   472
                     coset.coset_join2 [symmetric])
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   473
done
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   474
*)
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   475
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   476
lemma (in group) setrcos_inv_mult_group_eq:
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   477
     "[|H <| G; M \<in> rcosets G H|] ==> set_inv G M <#> M = H"
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   478
by (auto simp add: setrcos_eq rcos_inv rcos_sum normal_imp_subgroup
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   479
                   subgroup.subset)
13940
c67798653056 HOL-Algebra: New polynomial development added.
ballarin
parents: 13936
diff changeset
   480
(*
13889
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   481
lemma (in group) factorgroup_is_magma:
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   482
  "H <| G ==> magma (G Mod H)"
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   483
  by rule (simp add: FactGroup_def coset.setmult_closed [OF is_coset])
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   484
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   485
lemma (in group) factorgroup_semigroup_axioms:
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   486
  "H <| G ==> semigroup_axioms (G Mod H)"
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   487
  by rule (simp add: FactGroup_def coset.setrcos_assoc [OF is_coset]
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   488
    coset.setmult_closed [OF is_coset])
13940
c67798653056 HOL-Algebra: New polynomial development added.
ballarin
parents: 13936
diff changeset
   489
*)
13889
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   490
theorem (in group) factorgroup_is_group:
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   491
  "H <| G ==> group (G Mod H)"
14666
65f8680c3f16 improved notation;
wenzelm
parents: 14651
diff changeset
   492
apply (simp add: FactGroup_def)
13936
d3671b878828 Greatly extended CRing. Added Module.
ballarin
parents: 13889
diff changeset
   493
apply (rule groupI)
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   494
    apply (simp add: setmult_closed)
13936
d3671b878828 Greatly extended CRing. Added Module.
ballarin
parents: 13889
diff changeset
   495
   apply (simp add: normal_imp_subgroup subgroup_in_rcosets)
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   496
  apply (simp add: restrictI setmult_closed setrcos_assoc)
13889
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   497
 apply (simp add: normal_imp_subgroup
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   498
                  subgroup_in_rcosets setrcos_mult_eq)
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   499
apply (auto dest: setrcos_inv_mult_group_eq simp add: setinv_closed)
13889
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   500
done
6676ac2527fa Fixed Coset.thy (proved theorem factorgroup_is_group).
ballarin
parents: 13870
diff changeset
   501
14747
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   502
lemma (in group) inv_FactGroup:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   503
     "N <| G ==> X \<in> carrier (G Mod N) ==> inv\<^bsub>G Mod N\<^esub> X = set_inv G X"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   504
apply (rule group.inv_equality [OF factorgroup_is_group]) 
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   505
apply (simp_all add: FactGroup_def setinv_closed 
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   506
    setrcos_inv_mult_group_eq group.intro [OF prems])
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   507
done
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   508
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   509
text{*The coset map is a homomorphism from @{term G} to the quotient group
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   510
  @{term "G Mod N"}*}
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   511
lemma (in group) r_coset_hom_Mod:
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   512
  assumes N: "N <| G"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   513
  shows "(r_coset G N) \<in> hom G (G Mod N)"
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   514
by (simp add: FactGroup_def rcosets_def Pi_def hom_def
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   515
           rcos_sum group.intro prems) 
2eaff69d3d10 removal of locale coset
paulson
parents: 14706
diff changeset
   516
13870
cf947d1ec5ff moved Exponent, Coset, Sylow from GroupTheory to Algebra, converting them
paulson
parents:
diff changeset
   517
end