Existence of bases for crystallographic root systems #
Implementation details #
The proof needs a set of ordered coefficients, even though the ultimate existence statement does
not. There are at least two ways to deal with this:
(a) Using the fact that a crystallographic root system induces a ℚ-structure, pass to the root
system over ℚ defined by RootPairing.restrictScalarsRat, and develop a theory of base
change for root system bases.
(b) Introduce a second set of ordered coefficients (ultimately taken to be ℚ) and develop a
theory with two sets of coefficients simultaneously in play.
It is not really clear which is the better approach but here we opt for approach (b) as it seems to yield slightly more general results.
TODO #
- Prove that for crystallographic reduced root systems, the axiom
coroot_mem_or_neg_memappearing inRootPairing.Basefollows from the others, and combine this withRootPairing.linearIndepOn_coroot_iffto thus provide an alternate constructor forRootPairing.Basewhich demands only the hypotheses on the roots. - [Easy given 1 above] Prove that every reduced crystallographic root system has a base by
combining the constructor in 1 above with
RootPairing.linearIndepOn_root_baseOf,IsAddIndecomposable.mem_or_neg_mem_closure_baseOf,Module.exists_dual_forall_apply_ne_zero.
This is [Ser87](Ch. V, §9, Lemma 3).
This lemma is usually established for root systems with coefficients R equal to ℚ or ℝ, in
which case one may take S = R. However our statement allows for more general coefficients such as
R = ℂ and S = ℚ.
This lemma is mostly a stepping stone en route to RootPairing.linearIndepOn_root_baseOf (where
linear independence is established over R rather than just S) except that this version does not
make the field assumption and so covers the case S = R = ℤ which the latter does not.
A set of linearly independent roots whose cone span over ℕ contains all the roots is a basis
for the ambient space.
Equations
- P.basisOfBase s hli hsp = Module.Basis.mk hli ⋯