Skip to content

Commit

Permalink
feat: vectorSpan k (v +ᵥ s) = vectorSpan k s (#21305)
Browse files Browse the repository at this point in the history
From PFR
  • Loading branch information
YaelDillies authored and jt496 committed Feb 3, 2025
1 parent c970352 commit 68196da
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions Mathlib/LinearAlgebra/AffineSpace/AffineSubspace.lean
Original file line number Diff line number Diff line change
Expand Up @@ -90,6 +90,9 @@ theorem vsub_mem_vectorSpan {s : Set P} {p1 p2 : P} (hp1 : p1 ∈ s) (hp2 : p2
p1 -ᵥ p2 ∈ vectorSpan k s :=
vsub_set_subset_vectorSpan k s (vsub_mem_vsub hp1 hp2)

@[simp] lemma vectorSpan_vadd (s : Set P) (v : V) : vectorSpan k (v +ᵥ s) = vectorSpan k s := by
simp [vectorSpan]

/-- The points in the affine span of a (possibly empty) set of points. Use `affineSpan` instead to
get an `AffineSubspace k P`. -/
def spanPoints (s : Set P) : Set P :=
Expand Down

0 comments on commit 68196da

Please sign in to comment.