Skip to content

Commit 229276c

Browse files
committed
feat: vectorSpan k (v +ᵥ s) = vectorSpan k s (#21305)
From PFR
1 parent 5c57f97 commit 229276c

File tree

1 file changed

+3
-0
lines changed

1 file changed

+3
-0
lines changed

Mathlib/LinearAlgebra/AffineSpace/AffineSubspace.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -90,6 +90,9 @@ theorem vsub_mem_vectorSpan {s : Set P} {p1 p2 : P} (hp1 : p1 ∈ s) (hp2 : p2
9090
p1 -ᵥ p2 ∈ vectorSpan k s :=
9191
vsub_set_subset_vectorSpan k s (vsub_mem_vsub hp1 hp2)
9292

93+
@[simp] lemma vectorSpan_vadd (s : Set P) (v : V) : vectorSpan k (v +ᵥ s) = vectorSpan k s := by
94+
simp [vectorSpan]
95+
9396
/-- The points in the affine span of a (possibly empty) set of points. Use `affineSpan` instead to
9497
get an `AffineSubspace k P`. -/
9598
def spanPoints (s : Set P) : Set P :=

0 commit comments

Comments
 (0)