refactor: LInt
This commit is contained in:
parent
e963be5ef8
commit
d058f41689
11 changed files with 38 additions and 50 deletions
|
@ -10,7 +10,6 @@ import Mathlib.Algebra.Lie.Classical
|
|||
|
||||
# The Minkowski matrix
|
||||
|
||||
|
||||
-/
|
||||
|
||||
open Matrix
|
||||
|
@ -98,7 +97,6 @@ lemma mulVec_inr_i (v : (Fin 1 ⊕ Fin d) → ℝ) (i : Fin d) :
|
|||
simp only [mulVec, minkowskiMatrix, LieAlgebra.Orthogonal.indefiniteDiagonal, mulVec_diagonal]
|
||||
simp only [diagonal_dotProduct, Sum.elim_inr, neg_mul, one_mul]
|
||||
|
||||
|
||||
variable (Λ Λ' : Matrix (Fin 1 ⊕ Fin d) (Fin 1 ⊕ Fin d) ℝ)
|
||||
|
||||
/-- The dual of a matrix with respect to the Minkowski metric. -/
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue