Documentation

Mathlib.LinearAlgebra.Matrix.Charpoly.Univ

The universal characteristic polynomial #

In this file we define the universal characteristic polynomial Matrix.charpoly.univ, which is the charactistic polynomial of the matrix with entries Xᵢⱼ, and hence has coefficients that are multivariate polynomials.

It is universal in the sense that one obtains the characteristic polynomial of a matrix M by evaluating the coefficients of univ at the entries of M.

We use it to show that the coeffients of the characteristic polynomial of a matrix are homogeneous polynomials in the matrix entries.

Main results #

@[inline, reducible]
noncomputable abbrev Matrix.charpoly.univ (R : Type u_1) (n : Type u_3) [CommRing R] [Fintype n] [DecidableEq n] :

The universal characteristic polynomial for n × n-matrices, is the charactistic polynomial of Matrix.mvPolynomialX n n ℤ with entries Xᵢⱼ.

Its i-th coefficient is a homogeneous polynomial of degree n - i, see Matrix.charpoly.univ_coeff_isHomogeneous.

By evaluating the coefficients at the entries of a matrix M, one obtains the characteristic polynomial of M, see Matrix.charpoly.univ_map_eval₂Hom.

Equations
Instances For
    @[simp]
    theorem Matrix.charpoly.univ_map_eval₂Hom {R : Type u_1} {S : Type u_2} (n : Type u_3) [CommRing R] [CommRing S] [Fintype n] [DecidableEq n] (f : R →+* S) (M : n × nS) :
    @[simp]
    theorem Matrix.charpoly.univ_coeff_eval₂Hom {R : Type u_1} {S : Type u_2} (n : Type u_3) [CommRing R] [CommRing S] [Fintype n] [DecidableEq n] (f : R →+* S) (M : n × nS) (i : ) :