mathlib3 documentation

lean-ga / for_mathlib.linear_algebra.tensor_product.inner_product_space

@[simp]
theorem tmul_inner_tmul {V : Type u_1} {W : Type u_2} [normed_add_comm_group V] [normed_add_comm_group W] [inner_product_space V] [inner_product_space W] (v₁ : V) (w₁ : W) (v₂ : V) (w₂ : W) :
has_inner.inner (v₁ ⊗ₜ[] w₁) (v₂ ⊗ₜ[] w₂) = has_inner.inner v₁ v₂ * has_inner.inner w₁ w₂