Trace of a linear map #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines the trace of a linear map.
See also linear_algebra/matrix/trace.lean
for the trace of a matrix.
Tags #
linear_map, trace, diagonal
The trace of an endomorphism given a basis.
Equations
- linear_map.trace_aux R b = (matrix.trace_linear_map ι R R).comp ↑(linear_map.to_matrix b b)
Trace of an endomorphism independent of basis.
Auxiliary lemma for trace_eq_matrix_trace
.
The trace of an endomorphism is invariant under conjugation
The trace of a linear map correspond to the contraction pairing under the isomorphism
End(M) ≃ M* ⊗ M
The trace of a linear map correspond to the contraction pairing under the isomorphism
End(M) ≃ M* ⊗ M
When M
is finite free, the trace of a linear map correspond to the contraction pairing under
the isomorphism End(M) ≃ M* ⊗ M
When M
is finite free, the trace of a linear map correspond to the contraction pairing under
the isomorphism End(M) ≃ M* ⊗ M
The trace of the identity endomorphism is the dimension of the free module
The trace of the identity endomorphism is the dimension of the free module