Skip to content

Commit

Permalink
docs(RootSystem/Defs): add more details to the doc for root pairing…
Browse files Browse the repository at this point in the history
…s. (#19683)

Add a comparison with the "classical" literature in the definition of a root pairing.
  • Loading branch information
faenuccio committed Dec 2, 2024
1 parent 4587215 commit 7cf8077
Showing 1 changed file with 5 additions and 1 deletion.
6 changes: 5 additions & 1 deletion Mathlib/LinearAlgebra/RootSystem/Defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -92,7 +92,11 @@ structure RootPairing extends PerfectPairing R M N where
/-- A parametrized family of dual vectors, called coroots. -/
coroot : ι ↪ N
root_coroot_two : ∀ i, toLin (root i) (coroot i) = 2
/-- A parametrized family of permutations, induced by reflection. -/
/-- A parametrized family of permutations, induced by reflections. This corresponds to the
classical requirement that the symmetry attached to each root (later defined in
`RootPairing.reflection`) leave the whole set of roots stable: as explained above, we
formalize this stability by fixing the image of the roots through each reflection (whence the
permutation); and similarly for coroots. -/
reflection_perm : ι → (ι ≃ ι)
reflection_perm_root : ∀ i j,
root j - toPerfectPairing (root j) (coroot i) • root i = root (reflection_perm i j)
Expand Down

0 comments on commit 7cf8077

Please sign in to comment.