feat: Improved todo list
This commit is contained in:
parent
1b2cc5338f
commit
ca044d3786
37 changed files with 180 additions and 42 deletions
|
@ -8,6 +8,7 @@ import HepLean.Tensors.Tree.NodeIdentities.PermContr
|
|||
import HepLean.Tensors.Tree.NodeIdentities.ProdComm
|
||||
import HepLean.Tensors.Tree.NodeIdentities.ContrSwap
|
||||
import HepLean.Tensors.Tree.NodeIdentities.ContrContr
|
||||
import HepLean.Meta.TODO.Basic
|
||||
/-!
|
||||
|
||||
## Basis vectors associated with complex Lorentz tensors
|
||||
|
@ -47,7 +48,7 @@ lemma perm_basisVector_cast {n m : ℕ} {c : Fin n → complexLorentzTensor.C}
|
|||
simp only [Functor.const_obj_obj, OverColor.mk_hom] at h1
|
||||
rw [h1]
|
||||
|
||||
/-! TODO: Generalize `basis_eq_FD`. -/
|
||||
TODO "Generalize `basis_eq_FD`."
|
||||
lemma basis_eq_FD {n : ℕ} (c : Fin n → complexLorentzTensor.C)
|
||||
(b : Π j, Fin (complexLorentzTensor.repDim (c j))) (i : Fin n)
|
||||
(h : { as := c i } = { as := c1 }) :
|
||||
|
|
|
@ -388,7 +388,7 @@ lemma pauliMatrix_contr_lower_3_1_1 :
|
|||
· congr 2
|
||||
decide
|
||||
|
||||
/-! TODO: Work out why `pauliCo_prod_basis_expand'` is needed. -/
|
||||
TODO "Work out why `pauliCo_prod_basis_expand'` is needed."
|
||||
/-- This lemma is exactly the same as `pauliCo_prod_basis_expand`.
|
||||
It is needed here for `pauliMatrix_contract_pauliMatrix_aux`. It is unclear why
|
||||
`pauliMatrix_lower_basis_expand_prod` does not work. -/
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue