Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

Commit

Permalink
feat(linear_algebra/basis): repr_support_of_mem_span (#14504)
Browse files Browse the repository at this point in the history
This lemma states that if a vector is in the span of a subset of the basis vectors, only this subset of basis vectors will be used in its `repr` representation.



Co-authored-by: Alexander Bentkamp <a.bentkamp@vu.nl>
  • Loading branch information
abentkamp and abentkamp committed Jun 3, 2022
1 parent 2b69bb4 commit 31cbfbb
Showing 1 changed file with 7 additions and 0 deletions.
7 changes: 7 additions & 0 deletions src/linear_algebra/basis.lean
Original file line number Diff line number Diff line change
Expand Up @@ -146,6 +146,13 @@ lemma mem_span_repr_support {ι : Type*} (b : basis ι R M) (m : M) :
m ∈ span R (b '' (b.repr m).support) :=
(finsupp.mem_span_image_iff_total _).2 ⟨b.repr m, (by simp [finsupp.mem_supported_support])⟩

lemma repr_support_subset_of_mem_span {ι : Type*}
(b : basis ι R M) (s : set ι) {m : M} (hm : m ∈ span R (b '' s)) : ↑(b.repr m).support ⊆ s :=
begin
rcases (finsupp.mem_span_image_iff_total _).1 hm with ⟨l, hl, hlm⟩,
rwa [←hlm, repr_total, ←finsupp.mem_supported R l]
end

end repr

section coord
Expand Down

0 comments on commit 31cbfbb

Please sign in to comment.