feat: Improved todo list
This commit is contained in:
parent
1b2cc5338f
commit
ca044d3786
37 changed files with 180 additions and 42 deletions
|
@ -75,7 +75,7 @@ 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 "replace `Finsupp.equivFunOnFinite` here with `Finsupp.linearEquivFunOnFinite`."
|
||||
/-- The coordinate map for the basis. -/
|
||||
noncomputable
|
||||
def coordinateMap : (PureU1 n.succ).LinSols ≃ₗ[ℚ] Fin n →₀ ℚ where
|
||||
|
|
|
@ -616,7 +616,7 @@ lemma Pa'_eq (f f' : (Fin n.succ) ⊕ (Fin n) → ℚ) : Pa' f = Pa' f' ↔ f =
|
|||
linarith
|
||||
· rw [h]
|
||||
|
||||
/-! TODO: Replace the definition of `join` with a Mathlib definition, most likely `Sum.elim`. -/
|
||||
TODO "Replace the definition of `join` with a Mathlib definition, most likely `Sum.elim`."
|
||||
/-- A helper function for what follows. -/
|
||||
def join (g : Fin n.succ → ℚ) (f : Fin n → ℚ) : (Fin n.succ) ⊕ (Fin n) → ℚ := fun i =>
|
||||
match i with
|
||||
|
|
|
@ -623,7 +623,7 @@ lemma Pa'_eq (f f' : (Fin n.succ) ⊕ (Fin n.succ) → ℚ) : Pa' f = Pa' f' ↔
|
|||
linarith
|
||||
· rw [h]
|
||||
|
||||
/-! TODO: Replace the definition of `join` with a Mathlib definition, most likely `Sum.elim`. -/
|
||||
TODO "Replace the definition of `join` with a Mathlib definition, most likely `Sum.elim`."
|
||||
/-- A helper function for what follows. -/
|
||||
def join (g f : Fin n → ℚ) : Fin n ⊕ Fin n → ℚ := fun i =>
|
||||
match i with
|
||||
|
|
|
@ -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 "Replace the definition of `pairSwap` with `Equiv.swap`."
|
||||
/-- The permutation which swaps i and j. -/
|
||||
def pairSwap {n : ℕ} (i j : Fin n) : (FamilyPermutations n).group where
|
||||
toFun s :=
|
||||
|
|
|
@ -10,7 +10,7 @@ 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. -/
|
||||
TODO "Define vector like ACC in the `n`-odd case."
|
||||
universe v u
|
||||
|
||||
open Nat
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue