Documentation

Mathlib.LinearAlgebra.FreeModule.Finite.Matrix

Finite and free modules using matrices #

We provide some instances for finite and free modules involving matrices.

Main results #

instance Module.Free.linearMap (R : Type u) (S : Type u') (M : Type v) (N : Type w) [Ring R] [Ring S] [AddCommGroup M] [Module R M] [Free R M] [Module.Finite R M] [AddCommGroup N] [Module R N] [Module S N] [SMulCommClass R S N] [Free S N] :
Free S (M →ₗ[R] N)
instance Module.Finite.linearMap (R : Type u) (S : Type u') (M : Type v) (N : Type w) [Ring R] [Ring S] [AddCommGroup M] [Module R M] [Free R M] [Module.Finite R M] [AddCommGroup N] [Module R N] [Module S N] [SMulCommClass R S N] [Module.Finite S N] :
theorem Module.finrank_linearMap (R : Type u) (S : Type u') (M : Type v) (N : Type w) [Ring R] [Ring S] [AddCommGroup M] [Module R M] [Free R M] [Module.Finite R M] [AddCommGroup N] [Module R N] [Module S N] [SMulCommClass R S N] [StrongRankCondition R] [StrongRankCondition S] [Free S N] :
finrank S (M →ₗ[R] N) = finrank R M * finrank S N

The finrank of M →ₗ[R] N as an S-module is (finrank R M) * (finrank S N).

theorem Module.finrank_linearMap_self (R : Type u) (S : Type u') (M : Type v) [Ring R] [Ring S] [AddCommGroup M] [Module R M] [Free R M] [Module.Finite R M] [StrongRankCondition R] [StrongRankCondition S] [Module R S] [SMulCommClass R S S] :
finrank S (M →ₗ[R] S) = finrank R M
instance Finite.algHom (K : Type u_1) (M : Type u_2) (L : Type v) [CommRing K] [Ring M] [Algebra K M] [Module.Free K M] [Module.Finite K M] [CommRing L] [IsDomain L] [Algebra K L] :
@[deprecated cardinalMk_algHom_le_rank (since := "2024-11-10")]
theorem cardinal_mk_algHom_le_rank (K : Type u_1) (M : Type u_2) (L : Type v) [CommRing K] [Ring M] [Algebra K M] [Module.Free K M] [Module.Finite K M] [CommRing L] [IsDomain L] [Algebra K L] :

Alias of cardinalMk_algHom_le_rank.

theorem card_algHom_le_finrank (K : Type u_1) (M : Type u_2) (L : Type v) [CommRing K] [Ring M] [Algebra K M] [Module.Free K M] [Module.Finite K M] [CommRing L] [IsDomain L] [Algebra K L] :

Stacks Tag 09HS

theorem Matrix.rank_vecMulVec {K m n : Type u} [CommRing K] [Fintype n] [DecidableEq n] (w : mK) (v : nK) :
(toLin' (vecMulVec w v)).rank 1