refactor: Golfing

This commit is contained in:
jstoobysmith 2024-06-13 16:49:01 -04:00
parent d9f19aa028
commit 0346bf192b
9 changed files with 42 additions and 116 deletions

View file

@ -27,7 +27,7 @@ theorem solEqZero (S : (PureU1 1).LinSols) : S = 0 := by
simp at hLin
funext i
simp at i
rw [show i = (0 : Fin 1) by omega]
rw [show i = (0 : Fin 1) from Fin.fin_one_eq_zero i]
exact hLin
end One