refactor: Linting

This commit is contained in:
jstoobysmith 2024-07-30 08:07:47 -04:00
parent a65fb06605
commit a438af453d
14 changed files with 87 additions and 76 deletions

View file

@ -26,7 +26,6 @@ def rep : Representation (LorentzGroup d) (LorentzVector d) where
simp only [lorentzGroupIsGroup_mul_coe, map_mul]
open Matrix in
@[simp]
lemma rep_apply (g : LorentzGroup d) : rep g v = g *ᵥ v := rfl
end LorentzVector