feat: Add real lorentz tensors

This commit is contained in:
jstoobysmith 2024-07-29 16:54:59 -04:00
parent 44b26efdaf
commit 99f4e85839
13 changed files with 602 additions and 48 deletions

View file

@ -0,0 +1,30 @@
/-
Copyright (c) 2024 Joseph Tooby-Smith. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Joseph Tooby-Smith
-/
import HepLean.SpaceTime.LorentzVector.Basic
import HepLean.SpaceTime.LorentzGroup.Basic
import Mathlib.RepresentationTheory.Basic
/-!
# Lorentz group action on Lorentz vectors.
-/
noncomputable section
namespace LorentzVector
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_mul' x y := by
simp only [lorentzGroupIsGroup_mul_coe, map_mul]
end LorentzVector
end