Cartan matrices #
This file defines Cartan matrices for simple Lie algebras, both the exceptional types (E₆, E₇, E₈, F₄, G₂) and the classical infinite families (A, B, C, D).
Main definitions #
Exceptional types #
CartanMatrix.E₆: The Cartan matrix of type E₆CartanMatrix.E₇: The Cartan matrix of type E₇CartanMatrix.E₈: The Cartan matrix of type E₈CartanMatrix.F₄: The Cartan matrix of type F₄CartanMatrix.G₂: The Cartan matrix of type G₂
Classical types #
CartanMatrix.A: The Cartan matrix of type Aₙ₋₁ (corresponding to sl(n))CartanMatrix.B: The Cartan matrix of type Bₙ (corresponding to so(2n+1))CartanMatrix.C: The Cartan matrix of type Cₙ (corresponding to sp(2n))CartanMatrix.D: The Cartan matrix of type Dₙ (corresponding to so(2n))
References #
- N. Bourbaki, Lie Groups and Lie Algebras, Chapters 4--6 plates I -- IX
- [J. Humphreys, Introduction to Lie Algebras and Representation Theory] Chapter 11
Tags #
cartan matrix, lie algebra, dynkin diagram
Exceptional Cartan matrices #
The Cartan matrix of type E₆. See [Bou02] plate V, page 277.
Equations
- CartanMatrix.E₆ = !![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 F₄. See [Bou02] plate VIII, page 288.
Equations
- CartanMatrix.F₄ = !![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 [Bou02] plate IX, page 290. We use the transpose of Bourbaki's matrix for consistency with F₄.
Equations
- CartanMatrix.G₂ = !![2, -3; -1, 2]
Instances For
Classical Cartan matrices #
The Cartan matrix of type Bₙ (rank n, corresponding to so(2n+1)).
Equations
Instances For
Properties #
Transpose properties #
Small cases #
Exceptional matrix diagonal entries #
Exceptional matrix off-diagonal entries #
Exceptional matrix transpose properties #
Exceptional matrix determinants #
The determinants of E₆, E₇, E₈ are 3, 2, 1 respectively.
decide fails for these larger matrices without increasing the max recursion depth.
We could write manual proofs (e.g., expanding via det_succ_column_zero),
but prefer to wait for a more principled determinant tactic.
Equations
- One or more equations did not get rendered due to their size.
The Cartan matrices F₄ and G₂ are not simply laced because they contain off-diagonal entries that are neither 0 nor -1.