Apply the function f : α → β → γ
to each corresponding pair of elements from two vectors.
Equations
- List.Vector.zipWith f x y = ⟨List.zipWith f ↑x ↑y, ⋯⟩
Instances For
theorem
List.Vector.prod_mul_prod_eq_prod_zipWith
{α : Type u_1}
{n : ℕ}
[CommMonoid α]
(x y : Vector α n)
:
theorem
List.Vector.sum_add_sum_eq_sum_zipWith
{α : Type u_1}
{n : ℕ}
[AddCommMonoid α]
(x y : Vector α n)
: