refactor: Remove double empty lines
This commit is contained in:
parent
ae18a2196d
commit
f03d063c86
60 changed files with 0 additions and 232 deletions
|
@ -17,10 +17,8 @@ matrices.
|
|||
|
||||
-/
|
||||
|
||||
|
||||
noncomputable section
|
||||
|
||||
|
||||
open Matrix
|
||||
open Complex
|
||||
open ComplexConjugate
|
||||
|
@ -66,7 +64,6 @@ lemma not_orthochronous_iff_le_zero :
|
|||
rw [IsOrthochronous_iff_ge_one]
|
||||
linarith
|
||||
|
||||
|
||||
/-- The continuous map taking a Lorentz transformation to its `0 0` element. -/
|
||||
def timeCompCont : C(LorentzGroup d, ℝ) := ⟨fun Λ => timeComp Λ ,
|
||||
Continuous.matrix_elem (continuous_iff_le_induced.mpr fun _ a => a) (Sum.inl 0) (Sum.inl 0)⟩
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue