The span of a set of vectors, as a submodule #
Submodule.span sis defined to be the smallest submodule containing the sets.
Notation #
- We introduce the notation
R ∙ vfor the span of a singleton,Submodule.span R {v}. This is\span, not the same as the scalar multiplication•/\bub.
generator I, if I is a principal submodule, is an x ∈ M such that span R {x} = I
Equations
Instances For
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.
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.span_int_eq_addSubgroupClosure.
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_∙_» 70 70 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " ∙ ") (Lean.ParserDescr.cat `term 70))
Instances For
Unexpander for R ∙ x notation. This needs to be defined separately because the {_} notation is ambiguous, so we have to specify that it is the «term{_}» notation.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Alias of the forward direction of Submodule.codisjoint_iff_exists_add_eq.
Alias of Submodule.lt_sup_iff_notMem.
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.