feat: Add representations for real Lorentz vecs

This commit is contained in:
jstoobysmith 2024-11-08 06:54:55 +00:00
parent 6b6f9261ca
commit 87865a00b7
3 changed files with 42 additions and 1 deletions

View file

@ -35,7 +35,7 @@ namespace ContrModule
variable {d : }
/-- The equivalence between `ContrModule` and `Fin 1 ⊕ Fin d → `. -/
def toFin1dFun : ContrModule d ≃ (Fin 1 ⊕ Fin d → ) where
def toFin1dFun : ContrModule d ≃ (Fin 1 ⊕ Fin d → ) where
toFun v := v.val
invFun f := ⟨f⟩
left_inv _ := rfl