Calyley-Hamilton theorem for f.g. modules. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Given a fixed finite spanning set b : ι → M
of a R
-module M
, we say that a matrix M
represents an endomorphism f : M →ₗ[R] M
if the matrix as an endomorphism of ι → R
commutes
with f
via the projection (ι → R) →ₗ[R] M
given by b
.
We show that every endomorphism has a matrix representation, and if f.range ≤ I • ⊤
for some
ideal I
, we may furthermore obtain a matrix representation whose entries fall in I
.
This is used to conclude the Cayley-Hamilton theorem for f.g. modules over arbitrary rings.
The composition of a matrix (as an endomporphism of ι → R
) with the projection
(ι → R) →ₗ[R] M
.
Equations
- pi_to_module.from_matrix R b = (⇑(linear_map.llcomp R (ι → R) (ι → R) M) (⇑(fintype.total R R) b)).comp alg_equiv_matrix'.symm.to_linear_map
The endomorphisms of M
acts on (ι → R) →ₗ[R] M
, and takes the projection
to a (ι → R) →ₗ[R] M
.
Equations
- pi_to_module.from_End R b = linear_map.lcomp R M (⇑(fintype.total R R) b)
We say that a matrix represents an endomorphism of M
if the matrix acting on ι → R
is
equal to f
via the projection (ι → R) →ₗ[R] M
given by a fixed (spanning) set.
Equations
- matrix.represents b A f = (⇑(pi_to_module.from_matrix R b) A = ⇑(pi_to_module.from_End R b) f)
The subalgebra of matrix ι ι R
that consists of matrices that actually represent
endomorphisms on M
.
Equations
- matrix.is_representation R b = {carrier := {A : matrix ι ι R | ∃ (f : module.End R M), matrix.represents b A f}, mul_mem' := _, one_mem' := _, add_mem' := _, zero_mem' := _, algebra_map_mem' := _}
The map sending a matrix to the endomorphism it represents. This is an R
-algebra morphism.
Equations
- matrix.is_representation.to_End R b hb = {to_fun := λ (A : ↥(matrix.is_representation R b)), Exists.some _, map_one' := _, map_mul' := _, map_zero' := _, map_add' := _, commutes' := _}
The Cayley-Hamilton Theorem for f.g. modules over arbitrary rings states that for each
R
-endomorphism φ
of an R
-module M
such that φ(M) ≤ I • M
for some ideal I
, there
exists some n
and some aᵢ ∈ Iⁱ
such that φⁿ + a₁ φⁿ⁻¹ + ⋯ + aₙ = 0
.
This is the version found in Eisenbud 4.3, which is slightly weaker than Matsumura 2.1
(this lacks the constraint on n
), and is slightly stronger than Atiyah-Macdonald 2.4.