We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
vectorSpan k (v +ᵥ s) = vectorSpan k s
1 parent 5c57f97 commit 229276cCopy full SHA for 229276c
Mathlib/LinearAlgebra/AffineSpace/AffineSubspace.lean
@@ -90,6 +90,9 @@ theorem vsub_mem_vectorSpan {s : Set P} {p1 p2 : P} (hp1 : p1 ∈ s) (hp2 : p2
90
p1 -ᵥ p2 ∈ vectorSpan k s :=
91
vsub_set_subset_vectorSpan k s (vsub_mem_vsub hp1 hp2)
92
93
+@[simp] lemma vectorSpan_vadd (s : Set P) (v : V) : vectorSpan k (v +ᵥ s) = vectorSpan k s := by
94
+ simp [vectorSpan]
95
+
96
/-- The points in the affine span of a (possibly empty) set of points. Use `affineSpan` instead to
97
get an `AffineSubspace k P`. -/
98
def spanPoints (s : Set P) : Set P :=
0 commit comments