refactor: Improve todos and remove ambiguous

This commit is contained in:
jstoobysmith 2025-01-24 14:05:54 +00:00
parent 53476489c5
commit 944fabca1a
11 changed files with 25 additions and 15 deletions

View file

@ -75,7 +75,8 @@ lemma sum_of_vectors {n : } (f : Fin k → (PureU1 n).LinSols) (j : Fin n) :
(∑ i : Fin k, (f i)).1 j = (∑ i : Fin k, (f i).1 j) :=
sum_of_anomaly_free_linear (fun i => f i) j
TODO "replace `Finsupp.equivFunOnFinite` here with `Finsupp.linearEquivFunOnFinite`."
TODO "The definition of `coordinateMap` here may be improved by replacing
`Finsupp.equivFunOnFinite` with `Finsupp.linearEquivFunOnFinite`. Investigate this."
/-- The coordinate map for the basis. -/
noncomputable
def coordinateMap : (PureU1 n.succ).LinSols ≃ₗ[] Fin n →₀ where

View file

@ -89,7 +89,7 @@ lemma FamilyPermutations_anomalyFreeLinear_apply (S : (PureU1 n).LinSols)
((FamilyPermutations n).linSolRep f S).val i = S.val (f.invFun i) := by
rfl
TODO "Replace the definition of `pairSwap` with `Equiv.swap`."
TODO "Remove `pairSwap`, and use the Mathlib defined function `Equiv.swap` instead."
/-- The permutation which swaps i and j. -/
def pairSwap {n : } (i j : Fin n) : (FamilyPermutations n).group where
toFun s :=

View file

@ -10,7 +10,6 @@ import HepLean.AnomalyCancellation.PureU1.Sorts
For the `n`-even case we define the property of a charge assignment being vector like.
-/
TODO "Define vector like ACC in the `n`-odd case."
universe v u
open Nat