refactor: Replace simp proofs

This commit is contained in:
jstoobysmith 2024-08-30 13:40:32 -04:00
parent cd04e13ced
commit 064a5ebbfe
23 changed files with 110 additions and 148 deletions

View file

@ -20,8 +20,7 @@ variable {d : } (v : LorentzVector d)
/-- The contravariant action of the Lorentz group on a Lorentz vector. -/
def rep : Representation (LorentzGroup d) (LorentzVector d) where
toFun g := Matrix.toLinAlgEquiv e g
map_one' := by
simp only [lorentzGroupIsGroup_one_coe, map_one]
map_one' := (MulEquivClass.map_eq_one_iff (Matrix.toLinAlgEquiv e)).mpr rfl
map_mul' x y := by
simp only [lorentzGroupIsGroup_mul_coe, map_mul]