\( \newcommand\D{\mathrm{d}} \newcommand\E{\mathrm{e}} \newcommand\I{\mathrm{i}} \newcommand\bigOh{\mathcal{O}} \newcommand{\cat}[1]{\mathbf{#1}} \newcommand\curl{\vec{\nabla}\times} \newcommand{\CC}{\mathbb{C}} \newcommand{\NN}{\mathbb{N}} \newcommand{\QQ}{\mathbb{Q}} \newcommand{\RR}{\mathbb{R}} \newcommand{\ZZ}{\mathbb{Z}} \)
UP | HOME

Subgroup Series - Mizar

Table of Contents

1. Subgroup Series

I will review the various subgroup series, and — if they've been already defined (implicitly or explicitly) — their implementation.

1.1. Central Series

The definition of a nilpotent group uses a central series \(G=Z_{1}\geq Z_{2}\geq\dots\geq Z_{n}=\mathbf{1}\) where each \(Z_{k}\trianglelefteq G\) and the quotient satisfies \(Z_{k}/Z_{k+1}\leq Z(G/Z_{k+1})\).

definition
  let IT be Group;
  attr IT is nilpotent means :Def2: :: GRNILP_1:def 2
  ex F being FinSequence of the_normal_subgroups_of IT st
  (len F > 0 & F.1 = (Omega).IT & F.(len F) = (1).IT &
   (for i being Element of NAT st i in dom F & i+1 in dom F
    for G1, G2 being strict normal Subgroup of IT
    st G1 = F.i & G2 = F.(i + 1)
    holds (G2 is Subgroup of G1 &
           G1./.((G1,G2)`*`) is Subgroup of
             center (IT./.G2))));
end; 

1.2. Subnormal Series

A solvable group is defined by having a subnormal series \(G=N_{1}\trianglerighteq N_{2}\trianglerighteq\dots\trianglerighteq N_{n}=\mathbf{1}\) — that is, \(N_{j+1}\trianglelefteq N_{j}\) for \(j=0,\dots,n-1\) — whose factor groups \(N_{k}/N_{k+1}\) are Abelian.

definition
  let IT be Group;
  attr IT is solvable means :Def1: :: GRSOLV_1:def 1
  ex F being FinSequence of Subgroups IT st
  (len F > 0 & F.1 = (Omega).IT & F.(len F) = (1).IT &
   (for i being Element of NAT st i in dom F & i+1 in dom F
    for G1, G2 being strict Subgroup of IT
    st G1 = F.i & G2 = F.(i+1)
    holds (G2 is strict normal Subgroup of G1 &
           (for N being normal Subgroup of G1 st N = G2
            holds G1 ./. N is commutative))));
end; 

1.3. Composition Series

A famous example of a subgroup series is the composition series for a group. Mizar defines it as a subgroup series \(\mathbf{1}=A_{n}\trianglelefteq\dots\trianglelefteq A_{2}\trianglelefteq A_{1}=G\). Although this seems to be using a strange convention, Mizar is following Bourbaki's Algbra. The more familiar notion of a composition series (as a ``maximal'' subnormal series) requires the jordan_holder attribute (again, this follows Bourbaki's Algebra Definition 10 in I.4.7).

:: ALG I.4.7 Definition 9
definition
  let O be set;
  let G be GroupWithOperators of O;
  let IT be FinSequence of the_stable_subgroups_of G;
  attr IT is composition_series means
  :: GROUP_9:def 28
  IT.1=(Omega).G & IT.(len IT)= (1).G &
  for i being Nat st i in dom IT & i+1 in dom IT
  for H1,H2 being StableSubgroup of G
  st H1=IT.i & H2=IT.(i+1)
  holds H2 is normal StableSubgroup of H1;
end;

1.4. Lower Central Series

The lower central series may be defined as \(G=A_{1}\trianglerighteq A_{2}\trianglerighteq\dots\trianglerighteq A_{n}=\mathbf{1}\), where \(A_{k+1}=[A_{k},G]=[G,A_{k}]\). Mizar implicitly defines this in GRNILP1:Th27

theorem :: GRNILP_1:27
  for G being Group
  st ex F being FinSequence of the_normal_subgroups_of G
     st len F > 0 & F.1 = (Omega).G & F.(len F) = (1).G &
     for i st i in dom F & i+1 in dom F
     for G1 being strict normal Subgroup of G st G1 = F.i
     holds [.G1, (Omega).G.] = F.(i+1)
  holds G is nilpotent
proof end;

1.5. Upper Central Series

This is a subgroup series \(Z^0(G) \leq Z^1(G) \leq Z^2(G) \leq \dots\), where \(Z^{0}(G)=\mathbf{1}\), \(Z^1(G) = Z(G)\), \(Z^2(G)/Z^1(G) = Z(G/Z^1(G))\), \(Z^3(G)/Z^2(G) = Z(G/Z^2(G))\), and so on. Each \(Z^{n}(G)\) is a normal subgroup of \(G\).

In general, \(Z^{n+1}(G)/Z^{n}(G) = Z(G/Z^{n}(G))\) defines the \((n+1)\) term in the series. Explicitly, we would have

\[ Z^{n+1}(G) = \{x\in G\mid \forall y\in G, [x,y]\in Z^{n}(G)\}. \]

We could thus propose the definition (based on modifying the definition GRNILP_1:def 2 to use NAT_1 for mode sequence of X is Function of NAT,X):

definition
  let G be Group;
  func UpperCentralSeries G -> sequence of the_normal_subgroups_of G means
  :Def:
  (it.0 = (1).G &
   (for i being Element of NAT st i in dom it & i+1 in dom it
    for G1, G2 being strict normal Subgroup of G
    st G1 = it.i & G2 = it.(i + 1)
    holds (G1 is Subgroup of G2 &
           G2./.((G2,G1)`*`) = center (G./.G1))));
  existence
  proof
    thus ex Z being sequence of the_normal_subgroups_of G st
     (Z.0 = (1).G &
      (for i being Element of NAT st i in dom Z & i+1 in dom Z
       for G1, G2 being strict normal Subgroup of G
       st G1 = Z.i & G2 = Z.(i + 1)
       holds (G1 is Subgroup of G2 &
              G2./.((G2,G1)`*`) = center (G./.G1))));
  end;
  uniqueness
  proof
    defpred P[sequence of the_normal_subgroups_of G] means
    ($1.0 = (1).G &
      (for i being Element of NAT st i in dom $1 & i+1 in dom $1
       for G1, G2 being strict normal Subgroup of G
       st G1 = $1.i & G2 = $1.(i + 1)
       holds (G1 is Subgroup of G2 &
              G2./.((G2,G1)`*`) = center (G./.G1))));
    for Z1,Z2 being sequence of the_normal_subgroups_of G st
    P[Z1] & P[Z2] holds Z1=Z2;
    hence thesis;
  end;
end;

We would then have to prove

theorem
  for G be Group
  for n be Nat
  holds the carrier of (UpperCentralSeries G).(n+1) =
        {g where g is Element of G :
         for y being Element of G
         holds [.g,y.] in (UpperCentralSeries G).n};

Last Updated 2022-04-12 Tue 08:27.