refactor: Text based Lint
This commit is contained in:
parent
319089ad54
commit
7010a1dae2
12 changed files with 54 additions and 52 deletions
|
@ -209,10 +209,10 @@ 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} :
|
||||
instance {n : ℕ} {c : Fin n → complexLorentzTensor.C} :
|
||||
DecidableEq (OverColor.mk c).left := instDecidableEqFin n
|
||||
|
||||
instance {n : ℕ} {c : Fin n → complexLorentzTensor.C} :
|
||||
instance {n : ℕ} {c : Fin n → complexLorentzTensor.C} :
|
||||
Fintype (OverColor.mk c).left := Fin.fintype n
|
||||
|
||||
instance {n m : ℕ} {c : Fin n → complexLorentzTensor.C}
|
||||
|
@ -220,6 +220,5 @@ instance {n m : ℕ} {c : Fin n → complexLorentzTensor.C}
|
|||
Decidable (σ = σ') :=
|
||||
decidable_of_iff _ (OverColor.Hom.ext_iff σ σ')
|
||||
|
||||
|
||||
end complexLorentzTensor
|
||||
end
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue