mathlib documentation

linear_algebra.​char_poly.​coeff

linear_algebra.​char_poly.​coeff

Characteristic polynomials

We give methods for computing coefficients of the characteristic polynomial.

Main definitions

theorem char_matrix_apply_nat_degree {R : Type u} [comm_ring R] {n : Type v} [decidable_eq n] [fintype n] {M : matrix n n R} [nontrivial R] (i j : n) :
(char_matrix M i j).nat_degree = ite (i = j) 1 0

theorem char_matrix_apply_nat_degree_le {R : Type u} [comm_ring R] {n : Type v} [decidable_eq n] [fintype n] {M : matrix n n R} (i j : n) :
(char_matrix M i j).nat_degree ite (i = j) 1 0

theorem char_poly_sub_diagonal_degree_lt {R : Type u} [comm_ring R] {n : Type v} [decidable_eq n] [fintype n] (M : matrix n n R) :

theorem char_poly_coeff_eq_prod_coeff_of_le {R : Type u} [comm_ring R] {n : Type v} [decidable_eq n] [fintype n] (M : matrix n n R) {k : } :
fintype.card n - 1 k(char_poly M).coeff k = (finset.univ.prod (λ (i : n), polynomial.X - polynomial.C (M i i))).coeff k

theorem det_of_card_zero {R : Type u} [comm_ring R] {n : Type v} [decidable_eq n] [fintype n] (h : fintype.card n = 0) (M : matrix n n R) :
M.det = 1

theorem char_poly_degree_eq_dim {R : Type u} [comm_ring R] {n : Type v} [decidable_eq n] [fintype n] [nontrivial R] (M : matrix n n R) :

theorem char_poly_nat_degree_eq_dim {R : Type u} [comm_ring R] {n : Type v} [decidable_eq n] [fintype n] [nontrivial R] (M : matrix n n R) :

theorem char_poly_monic_of_nontrivial {R : Type u} [comm_ring R] {n : Type v} [decidable_eq n] [fintype n] [nontrivial R] (M : matrix n n R) :

theorem char_poly_monic {R : Type u} [comm_ring R] {n : Type v} [decidable_eq n] [fintype n] (M : matrix n n R) :

theorem trace_eq_neg_char_poly_coeff {R : Type u} [comm_ring R] {n : Type v} [decidable_eq n] [fintype n] [nonempty n] (M : matrix n n R) :

theorem mat_poly_equiv_eval {R : Type u} [comm_ring R] {n : Type v} [decidable_eq n] [fintype n] (M : matrix n n (polynomial R)) (r : R) (i j : n) :

theorem eval_det {R : Type u} [comm_ring R] {n : Type v} [decidable_eq n] [fintype n] (M : matrix n n (polynomial R)) (r : R) :

theorem det_eq_sign_char_poly_coeff {R : Type u} [comm_ring R] {n : Type v} [decidable_eq n] [fintype n] (M : matrix n n R) :