Zulip Chat Archive
Stream: mathlib4
Topic: Infoview no longer shows `*ᵥ`
Martin Dvořák (May 16 2024 at 06:37):
import Mathlib.LinearAlgebra.Matrix.DotProduct
open Matrix
example (A : Matrix (Fin 3) (Fin 2) ℚ) (v : Fin 2 → ℚ) : A *ᵥ v = A *ᵥ v := by
rfl
After switching to a new version, Infoview no longer shows *ᵥ
for Matrix.mulVec
— what happened?
Ruben Van de Velde (May 16 2024 at 07:47):
I think that's the dot notation issues that will be fixed in v4.8.0-rc2
Martin Dvořák (May 23 2024 at 07:19):
Yes, it has been fixed. Thanks!
Last updated: May 02 2025 at 03:31 UTC