Dot product of two vectors #
This file contains some results on the map matrix.dot_product
, which maps two
vectors v w : n → R
to the sum of the entrywise products v i * w i
.
Main results #
matrix.dot_product_std_basis_one
: the dot product ofv
with thei
th standard basis vector isv i
matrix.dot_product_eq_zero_iff
: ifv
's' dot product with allw
is zero, thenv
is zero
Tags #
matrix, reindex
@[simp]
theorem
matrix.dot_product_std_basis_eq_mul
{R : Type v}
[semiring R]
{n : Type w}
[fintype n]
[decidable_eq n]
(v : n → R)
(c : R)
(i : n) :
v ⬝ᵥ ⇑(linear_map.std_basis R (λ (_x : n), R) i) c = (v i) * c
@[simp]
theorem
matrix.dot_product_std_basis_one
{R : Type v}
[semiring R]
{n : Type w}
[fintype n]
[decidable_eq n]
(v : n → R)
(i : n) :
v ⬝ᵥ ⇑(linear_map.std_basis R (λ (_x : n), R) i) 1 = v i