refactor: Lint

This commit is contained in:
jstoobysmith 2024-07-02 10:26:21 -04:00
parent c64d926e7c
commit 304c3542b5
8 changed files with 10 additions and 29 deletions

View file

@ -4,7 +4,6 @@ Released under Apache 2.0 license.
Authors: Joseph Tooby-Smith
-/
import HepLean.SpaceTime.MinkowskiMetric
import HepLean.SpaceTime.LorentzVector.AsSelfAdjointMatrix
import HepLean.SpaceTime.LorentzVector.NormOne
/-!
# The Lorentz Group
@ -24,11 +23,8 @@ identity.
-/
noncomputable section
open Manifold
open Matrix
open Complex
open ComplexConjugate
@ -159,7 +155,6 @@ open minkowskiMetric
variable {Λ Λ' : LorentzGroup d}
@[simp]
lemma coe_inv : (Λ⁻¹).1 = Λ.1⁻¹:= by
refine (inv_eq_left_inv ?h).symm
exact mem_iff_dual_mul_self.mp Λ.2

View file

@ -21,7 +21,6 @@ matrices.
noncomputable section
open Manifold
open Matrix
open Complex
open ComplexConjugate

View file

@ -15,7 +15,6 @@ We define the give a series of lemmas related to the determinant of the lorentz
noncomputable section
open Manifold
open Matrix
open Complex
open ComplexConjugate