docs: More todos
This commit is contained in:
parent
b5a22f9685
commit
f83908e259
9 changed files with 13 additions and 23 deletions
|
@ -106,7 +106,8 @@ lemma FamilyPermutations_anomalyFreeLinear_apply (S : (PureU1 n).LinSols)
|
|||
((FamilyPermutations n).linSolRep f S).val i = S.val (f.invFun i) := by
|
||||
rfl
|
||||
|
||||
/-- The permutation which swaps i and j. TODO: Replace 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 :=
|
||||
if s = i then
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue