The span of a set of vectors, as a submodule #
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\span
, 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 = sInf {p : Submodule R M | s ⊆ ↑p}
Instances For
An R
-submodule of M
is principal if it is generated by one element.
- principal' : ∃ (a : M), S = Submodule.span R {a}
Instances
A version of Submodule.span_eq
for subobjects closed under addition and scalar multiplication
and containing zero. In general, this should not be used directly, but can be used to quickly
generate proofs for specific types of subobjects.
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
.
Alias of Submodule.span_induction
.
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
.
An induction principle for span membership. This is a version of Submodule.span_induction
for binary predicates.
A variant of span_induction
that combines ∀ x ∈ s, p x
and ∀ r x, p x → p (r • x)
into a single condition ∀ r, ∀ x ∈ s, p (r • x)
, which can be easier to verify.
Alias of Submodule.closure_induction
.
A variant of span_induction
that combines ∀ x ∈ s, p x
and ∀ r x, p x → p (r • x)
into a single condition ∀ r, ∀ x ∈ s, p (r • x)
, which can be easier to verify.
span
forms a Galois insertion with the coercion from submodule to set.
Equations
- Submodule.gi R M = { choice := fun (s : Set M) (x : ↑(Submodule.span R s) ≤ s) => Submodule.span R s, gc := ⋯, le_l_u := ⋯, choice_eq := ⋯ }
Instances For
Equations
- Submodule.«term_∙_» = Lean.ParserDescr.trailingNode `Submodule.«term_∙_» 1000 0 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " ∙ ") (Lean.ParserDescr.cat `term 0))
Instances For
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.