Documentation

Mathlib.Algebra.Lie.CartanMatrix

Lie algebras from Cartan matrices #

Split semi-simple Lie algebras are uniquely determined by their Cartan matrix. Indeed, if A is an l × l Cartan matrix, the corresponding Lie algebra may be obtained as the Lie algebra on 3l generators: $H_1, H_2, \ldots H_l, E_1, E_2, \ldots, E_l, F_1, F_2, \ldots, F_l$ subject to the following relations: $$ \begin{align} [H_i, H_j] &= 0\ [E_i, F_i] &= H_i\ [E_i, F_j] &= 0 \quad\text{if $i \ne j$}\ [H_i, E_j] &= A_{ij}E_j\ [H_i, F_j] &= -A_{ij}F_j\ ad(E_i)^{1 - A_{ij}}(E_j) &= 0 \quad\text{if $i \ne j$}\ ad(F_i)^{1 - A_{ij}}(F_j) &= 0 \quad\text{if $i \ne j$}\ \end{align} $$

In this file we provide the above construction. It is defined for any square matrix of integers but the results for non-Cartan matrices should be regarded as junk.

Recall that a Cartan matrix is a square matrix of integers A such that:

Alternative construction #

This construction is sometimes performed within the free unital associative algebra FreeAlgebra R X, rather than within the free Lie algebra FreeLieAlgebra R X, as we do here. However the difference is illusory since the construction stays inside the Lie subalgebra of FreeAlgebra R X generated by X, and this is naturally isomorphic to FreeLieAlgebra R X (though the proof of this seems to require Poincaré–Birkhoff–Witt).

Definitions of exceptional Lie algebras #

This file also contains the Cartan matrices of the exceptional Lie algebras. By using these in the above construction, it thus provides definitions of the exceptional Lie algebras. These definitions make sense over any commutative ring. When the ring is ℝ, these are the split real forms of the exceptional semisimple Lie algebras.

References #

Main definitions #

Tags #

lie algebra, semi-simple, cartan matrix

inductive CartanMatrix.Generators (B : Type v) :

The generators of the free Lie algebra from which we construct the Lie algebra of a Cartan matrix as a quotient.

Instances For

    The terms corresponding to the ⁅H, H⁆-relations.

    Equations
    Instances For

      The terms corresponding to the ⁅E, F⁆-relations.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For

        The terms corresponding to the ⁅H, E⁆-relations.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For

          The terms corresponding to the ⁅H, F⁆-relations.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For

            The terms corresponding to the ad E-relations.

            Note that we use Int.toNat so that we can take the power and that we do not bother restricting to the case i ≠ j since these relations are zero anyway. We also defensively ensure this with adE_of_eq_eq_zero.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For

              The terms corresponding to the ad F-relations.

              See also adE docstring.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For

                The union of all the relations as a subset of the free Lie algebra.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For

                  The ideal of the free Lie algebra generated by the relations.

                  Equations
                  Instances For
                    def Matrix.ToLieAlgebra (R : Type u) {B : Type v} [CommRing R] [DecidableEq B] (A : Matrix B B ) :
                    Type (max (max v u) u v)

                    The Lie algebra corresponding to a Cartan matrix.

                    Note that it is defined for any matrix of integers. Its value for non-Cartan matrices should be regarded as junk.

                    Equations
                    Instances For

                      The Cartan matrix of type e₆. See [bourbaki1968] plate V, page 277.

                      The corresponding Dynkin diagram is:

                                  o
                                  |
                      o --- o --- o --- o --- o
                      
                      Equations
                      • CartanMatrix.E₆ = Matrix.of ![![2, 0, -1, 0, 0, 0], ![0, 2, 0, -1, 0, 0], ![-1, 0, 2, -1, 0, 0], ![0, -1, -1, 2, -1, 0], ![0, 0, 0, -1, 2, -1], ![0, 0, 0, 0, -1, 2]]
                      Instances For

                        The Cartan matrix of type e₇. See [bourbaki1968] plate VI, page 281.

                        The corresponding Dynkin diagram is:

                                    o
                                    |
                        o --- o --- o --- o --- o --- o
                        
                        Equations
                        • One or more equations did not get rendered due to their size.
                        Instances For

                          The Cartan matrix of type e₈. See [bourbaki1968] plate VII, page 285.

                          The corresponding Dynkin diagram is:

                                      o
                                      |
                          o --- o --- o --- o --- o --- o --- o
                          
                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For

                            The Cartan matrix of type f₄. See [bourbaki1968] plate VIII, page 288.

                            The corresponding Dynkin diagram is:

                            o --- o =>= o --- o
                            
                            Equations
                            • CartanMatrix.F₄ = Matrix.of ![![2, -1, 0, 0], ![-1, 2, -2, 0], ![0, -1, 2, -1], ![0, 0, -1, 2]]
                            Instances For

                              The Cartan matrix of type g₂. See [bourbaki1968] plate IX, page 290.

                              The corresponding Dynkin diagram is:

                              o ≡>≡ o
                              

                              Actually we are using the transpose of Bourbaki's matrix. This is to make this matrix consistent with CartanMatrix.F₄, in the sense that all non-zero values below the diagonal are -1.

                              Equations
                              Instances For
                                @[inline, reducible]
                                abbrev LieAlgebra.e₆ (R : Type u) [CommRing R] :

                                The exceptional split Lie algebra of type e₆.

                                Equations
                                Instances For
                                  @[inline, reducible]
                                  abbrev LieAlgebra.e₇ (R : Type u) [CommRing R] :

                                  The exceptional split Lie algebra of type e₇.

                                  Equations
                                  Instances For
                                    @[inline, reducible]
                                    abbrev LieAlgebra.e₈ (R : Type u) [CommRing R] :

                                    The exceptional split Lie algebra of type e₈.

                                    Equations
                                    Instances For
                                      @[inline, reducible]
                                      abbrev LieAlgebra.f₄ (R : Type u) [CommRing R] :

                                      The exceptional split Lie algebra of type f₄.

                                      Equations
                                      Instances For
                                        @[inline, reducible]
                                        abbrev LieAlgebra.g₂ (R : Type u) [CommRing R] :

                                        The exceptional split Lie algebra of type g₂.

                                        Equations
                                        Instances For