feat: Fix pauli matrices as tensors. Speedup

This commit is contained in:
jstoobysmith 2024-10-25 13:50:19 +00:00
parent c565e7ea1c
commit e6ef68d7e6
9 changed files with 692 additions and 322 deletions

View file

@ -22,8 +22,8 @@ open TensorTree
open OverColor.Discrete
noncomputable section
namespace Fermion
open complexLorentzTensor
namespace complexLorentzTensor
open Fermion
set_option maxRecDepth 20000 in
lemma contr_rank_2_symm {T1 : (Lorentz.complexContr ⊗ Lorentz.complexContr).V}
{T2 : (Lorentz.complexCo ⊗ Lorentz.complexCo).V} :
@ -159,6 +159,6 @@ lemma leftMetric_mul_rightMetric_tree :
smul_tensor, neg_smul, one_smul]
rfl
end Fermion
end complexLorentzTensor
end