refactor: Linting substrings

This commit is contained in:
jstoobysmith 2024-07-12 16:22:06 -04:00
parent cee38b7be8
commit ac1132c7ca
40 changed files with 133 additions and 132 deletions

View file

@ -70,7 +70,7 @@ def mk₂ (f : V × V → ) (map_smul : ∀ a S T, f (a • S, T) = a * f (S,
simp only
rw [swap, map_add]
exact Mathlib.Tactic.LinearCombination.add_pf (swap T1 S) (swap T2 S)
map_smul' :=by
map_smul' := by
intro a T
simp only [eq_ratCast, Rat.cast_eq_id, id_eq, smul_eq_mul]
rw [swap, map_smul]
@ -173,7 +173,7 @@ namespace TriLinearSymm
open BigOperators
variable {V : Type} [AddCommMonoid V] [Module V]
instance instFun : FunLike (TriLinearSymm V) V (V →ₗ[] V →ₗ[] ) where
instance instFun : FunLike (TriLinearSymm V) V (V →ₗ[] V →ₗ[] ) where
coe f := f.toFun
coe_injective' f g h := by
cases f