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

@ -28,7 +28,7 @@ def equiv : (PureU1 2).LinSols ≃ (PureU1 2).Sols where
simp at hLin
erw [accCube_explicit]
simp only [Fin.sum_univ_two, Fin.isValue]
rw [show S.val (0 : Fin 2) = - S.val (1 : Fin 2) by linear_combination hLin]
rw [show S.val (0 : Fin 2) = - S.val (1 : Fin 2) from eq_neg_of_add_eq_zero_left hLin]
ring⟩
invFun S := S.1.1
left_inv S := rfl