feat: Einstein notation

This commit is contained in:
jstoobysmith 2024-08-15 13:52:50 -04:00
parent 7a5acb9734
commit f948f504c3
3 changed files with 92 additions and 1 deletions

View file

@ -86,7 +86,7 @@ instance : Fintype realTensorColor.Color := realTensorColor.instFintypeColorType
instance : DecidableEq realTensorColor.Color := realTensorColor.instDecidableEqColorType
/-! TODO: Set up the notation `𝓛𝓣` or similar. -/
/-- The `LorentzTensorStructure` associated with real Lorentz tensors. -/
/-- The `TensorStructure` associated with real Lorentz tensors. -/
def realLorentzTensor (d : ) : TensorStructure where
toTensorColor := realTensorColor
ColorModule μ :=
@ -146,4 +146,5 @@ instance : MulActionTensor (LorentzGroup d) (realLorentzTensor d) where
match μ with
| .up => asTenProd_invariant g
| .down => asCoTenProd_invariant g
end