Properties of the module α →₀ M #
Finsupp.linearEquivFunOnFinite:α →₀ βanda → βare equivalent ifαis finiteFunOnFinite.map: the map(X → M) → (Y → M)induced by a mapf : X ⟶ YwhenXandYare finite.FunOnFinite.linearMmap: the linear map(X → M) →ₗ[R] (Y → M)induced by a mapf : X ⟶ YwhenXandYare finite.
Tags #
function with finite support, module, linear algebra
If α has a unique term, then the type of finitely supported functions α →₀ M is
R-linearly equivalent to M.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Forget that a function is finitely supported.
This is the linear version of Finsupp.toFun.
Equations
- Finsupp.lcoeFun = { toFun := DFunLike.coe, map_add' := ⋯, map_smul' := ⋯ }
Instances For
A linear map from a product module P × M to M induces a linear map from P^(ℕ) to M,
where the nth component is given by P —ι₁→ P × M composed with P × M —f→ M —ι₂→ P × M
n times.
Equations
- f.prodOfFinsuppNat = (Finsupp.lsum ℕ) fun (n : ℕ) => ((LinearMap.inr R P M ∘ₗ f) ^ n) ∘ₗ LinearMap.inl R P M
Instances For
A surjective linear map to functions on a finite type has a splitting.
Equations
- f.splittingOfFunOnFintypeSurjective s = ((Finsupp.lift M R α) fun (x : α) => ⋯.choose) ∘ₗ ↑(Finsupp.linearEquivFunOnFinite R R α).symm
Instances For
Given a family Sᵢ of R-submodules of M indexed by a type α, this is the R-submodule
of α →₀ M of functions f such that f i ∈ Sᵢ for all i : α.
Equations
Instances For
The map (X → M) → (Y → M) induced by a map X → Y between finite types.
Equations
Instances For
The linear map (X → M) →ₗ[R] (Y → M) induced by a map X → Y between finite types.
Equations
- FunOnFinite.linearMap R M f = (↑(Finsupp.linearEquivFunOnFinite R M Y) ∘ₗ Finsupp.lmapDomain M R f) ∘ₗ ↑(Finsupp.linearEquivFunOnFinite R M X).symm