feat: Important fix to ContrContr
This commit is contained in:
parent
83ff8f5358
commit
4756466001
7 changed files with 184 additions and 2 deletions
|
@ -209,5 +209,17 @@ lemma basis_contr (c : complexLorentzTensor.C) (i : Fin (complexLorentzTensor.re
|
|||
| Color.up => Lorentz.contrCoContraction_basis _ _
|
||||
| Color.down => Lorentz.coContrContraction_basis _ _
|
||||
|
||||
instance {n : ℕ} {c : Fin n → complexLorentzTensor.C} :
|
||||
DecidableEq (OverColor.mk c).left := instDecidableEqFin n
|
||||
|
||||
instance {n : ℕ} {c : Fin n → complexLorentzTensor.C} :
|
||||
Fintype (OverColor.mk c).left := Fin.fintype n
|
||||
|
||||
instance {n m : ℕ} {c : Fin n → complexLorentzTensor.C}
|
||||
{c1 : Fin m → complexLorentzTensor.C} (σ σ' : OverColor.mk c ⟶ OverColor.mk c1) :
|
||||
Decidable (σ = σ') :=
|
||||
decidable_of_iff _ (OverColor.Hom.ext_iff σ σ')
|
||||
|
||||
|
||||
end complexLorentzTensor
|
||||
end
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue