refactor: Linting

This commit is contained in:
jstoobysmith 2024-07-18 16:46:29 -04:00
parent 1233987bd7
commit 52e591fa7a
27 changed files with 53 additions and 57 deletions

View file

@ -183,12 +183,11 @@ lemma QuadSols.ext {χ : ACCSystemQuad} {S T : χ.QuadSols} (h : S.val = T.val)
/-- An instance giving the properties and structures to define an action of `` on `QuadSols`. -/
instance quadSolsMulAction (χ : ACCSystemQuad) : MulAction χ.QuadSols where
smul a S := ⟨a • S.toLinSols , by
smul a S := ⟨a • S.toLinSols, by
intro i
erw [(χ.quadraticACCs i).map_smul]
rw [S.quadSol i]
simp only [mul_zero]
simp only [mul_zero]⟩
mul_smul a b S := by
apply QuadSols.ext
exact mul_smul _ _ _