Skip to content

Commit

Permalink
feat(LinearAlgebra): add Submodule.span_eq_top_of_restrictScalars (#…
Browse files Browse the repository at this point in the history
  • Loading branch information
erdOne committed Jan 25, 2025
1 parent efeadfb commit b3dcc0f
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions Mathlib/LinearAlgebra/Span/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -191,6 +191,9 @@ theorem span_span_of_tower :
span S (span R s : Set M) = span S s :=
le_antisymm (span_le.2 <| span_subset_span R S s) (span_mono subset_span)

theorem span_eq_top_of_span_eq_top (s : Set M) (hs : span R s = ⊤) : span S s = ⊤ :=
le_top.antisymm (hs.ge.trans (span_le_restrictScalars R S s))

variable {R S} in
lemma span_range_inclusion_eq_top (p : Submodule R M) (q : Submodule S M)
(h₁ : p ≤ q.restrictScalars R) (h₂ : q ≤ span S p) :
Expand Down

0 comments on commit b3dcc0f

Please sign in to comment.