refactor: Remove double empty lines
This commit is contained in:
parent
ae18a2196d
commit
f03d063c86
60 changed files with 0 additions and 232 deletions
|
@ -96,7 +96,6 @@ def FamilyPermutations (n : ℕ) : ACCSystemGroupAction (PureU1 n) where
|
|||
exact Fin.elim0 i
|
||||
cubicInvariant := accCube_invariant
|
||||
|
||||
|
||||
lemma FamilyPermutations_charges_apply (S : (PureU1 n).Charges)
|
||||
(i : Fin n) (f : (FamilyPermutations n).group) :
|
||||
((FamilyPermutations n).rep f S) i = S (f.invFun i) := by
|
||||
|
@ -107,7 +106,6 @@ 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`. -/
|
||||
def pairSwap {n : ℕ} (i j : Fin n) : (FamilyPermutations n).group where
|
||||
toFun s :=
|
||||
|
@ -247,7 +245,6 @@ lemma permThreeInj_fst_apply :
|
|||
⟨i, permThreeInj_fst hij hjk hik⟩ = 0 := by
|
||||
exact (Equiv.symm_apply_eq (Function.Embedding.toEquivRange (permThreeInj hij hjk hik))).mpr rfl
|
||||
|
||||
|
||||
lemma permThreeInj_snd : j ∈ Set.range ⇑(permThreeInj hij hjk hik) := by
|
||||
simp only [Set.mem_range]
|
||||
use 1
|
||||
|
@ -338,5 +335,4 @@ lemma Prop_three (P : ℚ × ℚ × ℚ → Prop) {S : (PureU1 n).LinSols}
|
|||
erw [permThree_fst,permThree_snd, permThree_thd] at h1
|
||||
exact h1
|
||||
|
||||
|
||||
end PureU1
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue