refactor: More simps

This commit is contained in:
jstoobysmith 2024-10-12 08:42:20 +00:00
parent 4a396783ab
commit 269f4d53a7
16 changed files with 139 additions and 62 deletions

View file

@ -35,7 +35,7 @@ def BL₁ : (PlusU1 1).Sols where
| (5 : Fin 6) => 3
linearSol := by
intro i
simp at i
simp only [PlusU1_numberLinear] at i
match i with
| 0 => rfl
| 1 => rfl
@ -43,7 +43,7 @@ def BL₁ : (PlusU1 1).Sols where
| 3 => rfl
quadSol := by
intro i
simp at i
simp only [PlusU1_numberQuadratic] at i
match i with
| 0 => rfl
cubicSol := by rfl