Bases for root pairings / systems #
This file contains a theory of bases for root pairings / systems.
Implementation details #
For reduced root pairings RootSystem.Base
is equivalent to the usual definition appearing in the
informal literature (e.g., it follows from [Ser87](Ch. V, §8, Proposition 7) that
RootSystem.Base
is equivalent to both [Ser87](Ch. V, §8, Definition 5) and
[Bou02](Ch. VI, §1.5) for reduced pairings). However for non-reduced root pairings, it is
more restrictive because it includes axioms on coroots as well as on roots. For example by
RootPairing.Base.eq_one_or_neg_one_of_mem_support_of_smul_mem
it is clear that the 1-dimensional
root system {-2, -1, 0, 1, 2} ⊆ ℝ
has no base in the sense of RootSystem.Base
.
It is also worth remembering that it is only for reduced root systems that one has the simply transitive action of the Weyl group on the set of bases, and that the Weyl group of a non-reduced root system is the same as that of the reduced root system obtained by passing to the indivisible roots.
For infinite root systems, RootSystem.Base
is usually not the right notion: linear independence
is too strong.
Main definitions / results: #
RootSystem.Base
: a base of a root pairing.RootSystem.Base.IsPos
: the predicate that a (co)root is positive relative to a base.RootSystem.Base.induction_add
: an induction principle for predicates on (co)roots which respect addition of a simple root.RootSystem.Base.induction_reflect
: an induction principle for predicates on (co)roots which respect reflection in a simple root.
TODO #
- Develop a theory of base / separation / positive roots for infinite systems which specialises to the concept here for finite systems.
A base of a root pairing.
For reduced root pairings this definition is equivalent to the usual definition appearing in the informal literature but not for non-reduced root pairings it is more restrictive. See the module doc string for further remarks.
- support : Finset ι
The indices of the simple roots / coroots.
- linearIndepOn_root : LinearIndepOn R ⇑P.root ↑self.support
- linearIndepOn_coroot : LinearIndepOn R ⇑P.coroot ↑self.support
Instances For
Interchanging roots and coroots, one still has a base of a root pairing.
Equations
Instances For
Alias of RootPairing.Base.sub_notMem_range_root
.
Alias of RootPairing.Base.sub_notMem_range_coroot
.
A base of a root system yields a basis of the root space.
Equations
- b.toWeightBasis = Basis.mk ⋯ ⋯
Instances For
A base of a root system yields a basis of the coroot space.
Equations
Instances For
Given a base α₁, α₂, …
, the height of a root ∑ zᵢαᵢ
relative to this base is ∑ zᵢ
.
Instances For
The predicate that a (co)root is positive with respect to a base.
Instances For
This lemma is included mostly for comparison with the informal literature. Usually
RootPairing.Base.IsPos.induction_on_add
will be more useful.