Skip to content

Commit

Permalink
feat(linear_algebra/affine_space/affine_subspace): `vector_span_inser…
Browse files Browse the repository at this point in the history
…t_eq_vector_span` (#16765)

Add a variant of `affine_span_insert_eq_affine_span` for the `vector_span`.
  • Loading branch information
jsm28 committed Oct 3, 2022
1 parent 81120ae commit 64b6d04
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/linear_algebra/affine_space/affine_subspace.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1161,6 +1161,14 @@ begin
rw [←affine_span_insert_affine_span, set.insert_eq_of_mem h, affine_span_coe]
end

variables {k}

/-- If a point is in the affine span of a set, adding it to that set
does not change the vector span. -/
lemma vector_span_insert_eq_vector_span {p : P} {ps : set P} (h : p ∈ affine_span k ps) :
vector_span k (insert p ps) = vector_span k ps :=
by simp_rw [←direction_affine_span, affine_span_insert_eq_affine_span _ h]

end affine_space'

namespace affine_subspace
Expand Down

0 comments on commit 64b6d04

Please sign in to comment.