refactor: Fix imports and some lint

This commit is contained in:
jstoobysmith 2024-10-19 08:49:26 +00:00
parent 14bf127335
commit b2ac704d80
14 changed files with 47 additions and 69 deletions

View file

@ -34,10 +34,6 @@ open Matrix
example (v : Fermion.leftHanded) : TensorTree complexLorentzTensor ![Color.upL] :=
{v | i}ᵀ
example (v : Fermion.leftHanded ⊗ Lorentz.complexContr) :
TensorTree complexLorentzTensor ![Color.upL, Color.up] :=
{v | i j}ᵀ
example :
TensorTree complexLorentzTensor ![Color.downR, Color.downR] :=
{Fermion.altRightMetric | μ j}ᵀ
@ -55,13 +51,13 @@ open Lean.Elab
open Lean.Elab.Term
open Lean Meta Elab Tactic
open IndexNotation
/-
example : True :=
let f := {Lorentz.coMetric | μ ν ⊗ PauliMatrix.asConsTensor | μ α β ⊗ PauliMatrix.asConsTensor | ν α' β'}ᵀ
have h1 : {Lorentz.coMetric | μ ν = Lorentz.coMetric | μ ν}ᵀ := by
sorry
sorry
-/
end Fermion
end

View file

@ -67,8 +67,7 @@ lemma coMetric_symm : {Lorentz.coMetric | μ ν = Lorentz.coMetric | ν μ}ᵀ :
| (0 : Fin 2) => rfl
| (1 : Fin 2) => rfl
open TensorTree in
/-
lemma coMetric_prod_antiSymm (A : (Lorentz.complexContr ⊗ Lorentz.complexContr).V)
(S : (Lorentz.complexCo ⊗ Lorentz.complexCo).V)
(hA : (twoNodeE complexLorentzTensor Color.up Color.up A).tensor =
@ -85,7 +84,7 @@ lemma coMetric_prod_antiSymm (A : (Lorentz.complexContr ⊗ Lorentz.complexContr
apply congrArg
sorry
sorry
-/
end Fermion
end