Characteristic polynomials of linear families of endomorphisms #
The coefficients of the characteristic polynomials of a linear family of endomorphisms are homogeneous polynomials in the parameters. This result is used in Lie theory to establish the existence of regular elements and Cartan subalgebras, and ultimately a well-defined notion of rank for Lie algebras.
In this file we prove this result about characteristic polynomials.
Let L
and M
be modules over a nontrivial commutative ring R
,
and let φ : L →ₗ[R] Module.End R M
be a linear map.
Let b
be a basis of L
, indexed by ι
.
Then we define a multivariate polynomial with variables indexed by ι
that evaluates on elements x
of L
to the characteristic polynomial of φ x
.
Main declarations #
Matrix.toMvPolynomial M i
: the family of multivariate polynomials that evaluates onc : n → R
to the dot product of thei
-th row ofM
withc
.Matrix.toMvPolynomial M i
is the sum of the monomialsC (M i j) * X j
.LinearMap.toMvPolynomial b₁ b₂ f
: a version ofMatrix.toMvPolynomial
for linear mapsf
with respect to basesb₁
andb₂
of the domain and codomain.LinearMap.polyCharpoly
: the multivariate polynomial that evaluates on elementsx
ofL
to the characteristic polynomial ofφ x
.LinearMap.polyCharpoly_map_eq_charpoly
: the evaluation ofpolyCharpoly
on elementsx
ofL
is the characteristic polynomial ofφ x
.LinearMap.polyCharpoly_coeff_isHomogeneous
: the coefficients ofpolyCharpoly
are homogeneous polynomials in the parameters.LinearMap.nilRank
: the smallest index at whichpolyCharpoly
has a non-zero coefficient, which is independent of the choice of basis forL
.LinearMap.IsNilRegular
: an elementx
ofL
is nil-regular with respect toφ
if then
-th coefficient of the characteristic polynomial ofφ x
is non-zero, wheren
denotes the nil-rank ofφ
.
Implementation details #
We show that LinearMap.polyCharpoly
does not depend on the choice of basis of the target module.
This is done via LinearMap.polyCharpoly_eq_polyCharpolyAux
and LinearMap.polyCharpolyAux_basisIndep
.
The latter is proven by considering
the base change of the R
-linear map φ : L →ₗ[R] End R M
to the multivariate polynomial ring MvPolynomial ι R
,
and showing that polyCharpolyAux φ
is equal to the characteristic polynomial of this base change.
The proof concludes because characteristic polynomials are independent of the chosen basis.
References #
- [Bar67]: "On Cartan subalgebras of Lie algebras" by D.W. Barnes.
Let M
be an (m × n)
-matrix over R
.
Then Matrix.toMvPolynomial M
is the family (indexed by i : m
)
of multivariate polynomials in n
variables over R
that evaluates on c : n → R
to the dot product of the i
-th row of M
with c
:
Matrix.toMvPolynomial M i
is the sum of the monomials C (M i j) * X j
.
Equations
- M.toMvPolynomial i = ∑ j : n, (MvPolynomial.monomial (Finsupp.single j 1)) (M i j)
Instances For
Let f : M₁ →ₗ[R] M₂
be an R
-linear map
between modules M₁
and M₂
with bases b₁
and b₂
respectively.
Then LinearMap.toMvPolynomial b₁ b₂ f
is the family of multivariate polynomials over R
that evaluates on an element x
of M₁
(represented on the basis b₁
)
to the element f x
of M₂
(represented on the basis b₂
).
Equations
- LinearMap.toMvPolynomial b₁ b₂ f i = ((LinearMap.toMatrix b₁ b₂) f).toMvPolynomial i
Instances For
(Implementation detail, see LinearMap.polyCharpoly
.)
Let L
and M
be finite free modules over R
,
and let φ : L →ₗ[R] Module.End R M
be a linear map.
Let b
be a basis of L
and bₘ
a basis of M
.
Then LinearMap.polyCharpolyAux φ b bₘ
is the polynomial that evaluates on elements x
of L
to the characteristic polynomial of φ x
acting on M
.
This definition does not depend on the choice of bₘ
(see LinearMap.polyCharpolyAux_basisIndep
).
Equations
- φ.polyCharpolyAux b bₘ = Polynomial.map (↑(MvPolynomial.bind₁ (LinearMap.toMvPolynomial b bₘ.end φ))) (Matrix.charpoly.univ R ιM)
Instances For
LinearMap.polyCharpolyAux
is independent of the choice of basis of the target module.
Proof strategy:
- Rewrite
polyCharpolyAux
as the (honest, ordinary) characteristic polynomial of the basechange ofφ
to the multivariate polynomial ringMvPolynomial ι R
. - Use that the characteristic polynomial of a linear map is independent of the choice of basis.
This independence result is used transitively via
LinearMap.polyCharpolyAux_map_aeval
andLinearMap.polyCharpolyAux_map_eq_charpoly
.
Let L
and M
be finite free modules over R
,
and let φ : L →ₗ[R] Module.End R M
be a linear family of endomorphisms.
Let b
be a basis of L
and bₘ
a basis of M
.
Then LinearMap.polyCharpoly φ b
is the polynomial that evaluates on elements x
of L
to the characteristic polynomial of φ x
acting on M
.
Equations
- φ.polyCharpoly b = φ.polyCharpolyAux b (Module.Free.chooseBasis R M)
Instances For
(Implementation detail, see LinearMap.nilRank
.)
Let L
and M
be finite free modules over R
,
and let φ : L →ₗ[R] Module.End R M
be a linear family of endomorphisms.
Then LinearMap.nilRankAux φ b
is the smallest index
at which LinearMap.polyCharpoly φ b
has a non-zero coefficient.
This number does not depend on the choice of b
, see nilRankAux_basis_indep
.
Equations
- φ.nilRankAux b = (φ.polyCharpoly b).natTrailingDegree
Instances For
Let L
and M
be finite free modules over R
,
and let φ : L →ₗ[R] Module.End R M
be a linear family of endomorphisms.
Then LinearMap.nilRank φ b
is the smallest index
at which LinearMap.polyCharpoly φ b
has a non-zero coefficient.
This number does not depend on the choice of b
,
see LinearMap.nilRank_eq_polyCharpoly_natTrailingDegree
.
Equations
- φ.nilRank = φ.nilRankAux (Module.Free.chooseBasis R L)
Instances For
Let L
and M
be finite free modules over R
,
and let φ : L →ₗ[R] Module.End R M
be a linear family of endomorphisms,
and denote n := nilRank φ
.
An element x : L
is nil-regular with respect to φ
if the n
-th coefficient of the characteristic polynomial of φ x
is non-zero.
Equations
- φ.IsNilRegular x = ((LinearMap.charpoly (φ x)).coeff φ.nilRank ≠ 0)