feat: Make MulActionTensor

This commit is contained in:
jstoobysmith 2024-07-30 07:51:07 -04:00
parent 99f4e85839
commit a65fb06605
11 changed files with 177 additions and 55 deletions

View file

@ -25,6 +25,10 @@ def rep : Representation (LorentzGroup d) (LorentzVector d) where
map_mul' x y := by
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
end