refactor: Lint

This commit is contained in:
jstoobysmith 2024-11-10 06:57:41 +00:00
parent 6c17a61989
commit b0c5ed894f
8 changed files with 16 additions and 11 deletions

View file

@ -61,9 +61,6 @@ def Co (d : ) : Rep (LorentzGroup d) := Rep.of CoMod.rep
open CategoryTheory.MonoidalCategory
def toField (d : ) : (𝟙_ (Rep ↑(LorentzGroup d))) →ₗ[] := LinearMap.id
lemma toField_apply {d : } (a : 𝟙_ (Rep ↑(LorentzGroup d))) : toField d a = a := rfl
/-!
## Isomorphism between contravariant and covariant Lorentz vectors