The span of a set of vectors, as a submodule #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
submodule.span s
is defined to be the smallest submodule containing the sets
.
Notations #
- We introduce the notation
R ∙ v
for the span of a singleton,submodule.span R {v}
. This is\.
, not the same as the scalar multiplication•
/\bub
.
The span of a set s ⊆ M
is the smallest submodule of M that contains s
.
Equations
- submodule.span R s = has_Inf.Inf {p : submodule R M | s ⊆ ↑p}
Instances for ↥submodule.span
A version of submodule.span_eq
for when the span is by a smaller ring.
Alias of submodule.map_span
.
Alias of submodule.map_span_le
.
Alias of submodule.span_preimage_le
.
An induction principle for span membership. If p
holds for 0 and all elements of s
, and is
preserved under addition and scalar multiplication, then p
holds for all elements of the span of
s
.
A dependent version of submodule.span_induction
.
span
forms a Galois insertion with the coercion from submodule to set.
Equations
- submodule.gi R M = {choice := λ (s : set M) (_x : ↑(submodule.span R s) ≤ s), submodule.span R s, gc := _, le_l_u := _, choice_eq := _}
See submodule.span_smul_eq
(in ring_theory.ideal.operations
) for
span R (r • s) = r • span R s
that holds for arbitrary r
in a comm_semiring
.
We can regard coe_supr_of_chain
as the statement that coe : (submodule R M) → set M
is
Scott continuous for the ω-complete partial order induced by the complete lattice structures.
If R
is "smaller" ring than S
then the span by R
is smaller than the span by S
.
A version of submodule.span_le_restrict_scalars
with coercions.
Taking the span by a large ring of the span by the small ring is the same as taking the span by just the large ring.
f
is an explicit argument so we can apply
this theorem and obtain h
as a new goal.
An induction principle for elements of ⨆ i, p i
.
If C
holds for 0
and all elements of p i
for all i
, and is preserved under addition,
then it holds for all elements of the supremum of p
.
A dependent version of submodule.supr_induction
.
The span of a finite subset is compact in the lattice of submodules.
The span of a finite subset is compact in the lattice of submodules.
A submodule is equal to the supremum of the spans of the submodule's nonzero elements.
For every element in the span of a set, there exists a finite subset of the set such that the element is contained in the span of the subset.
The product of two submodules is a submodule.
Given an element x
of a module M
over R
, the natural map from
R
to scalar multiples of x
.
Equations
The range of to_span_singleton x
is the span of x
.
If two linear maps are equal on a set s
, then they are equal on submodule.span s
.
See also linear_map.eq_on_span'
for a version using set.eq_on
.
If two linear maps are equal on a set s
, then they are equal on submodule.span s
.
This version uses set.eq_on
, and the hidden argument will expand to h : x ∈ (span R s : set M)
.
See linear_map.eq_on_span
for a version that takes h : x ∈ span R s
as an argument.
If s
generates the whole module and linear maps f
, g
are equal on s
, then they are
equal.
If the range of v : ι → M
generates the whole module and linear maps f
, g
are equal at
each v i
, then they are equal.
Given a nonzero element x
of a torsion-free module M
over a ring R
, the natural
isomorphism from R
to the span of x
given by $r \mapsto r \cdot x$.
Equations
- linear_equiv.to_span_nonzero_singleton R M x h = (linear_equiv.of_injective (linear_map.to_span_singleton R M x) _).trans (linear_equiv.of_eq (linear_map.range (linear_map.to_span_singleton R M x)) (submodule.span R {x}) _)
Given a nonzero element x
of a torsion-free module M
over a ring R
, the natural
isomorphism from the span of x
to R
given by $r \cdot x \mapsto r$.