chore: Double line linter

This commit is contained in:
jstoobysmith 2024-07-03 07:41:06 -04:00
parent bd9f796110
commit ae18a2196d
8 changed files with 75 additions and 17 deletions

View file

@ -70,14 +70,11 @@ def accCubeTriLinSymm {n : } : TriLinearSymm (PureU1Charges n).Charges := Tri
ring
)
/-- The cubic anomaly equation. -/
@[simp]
def accCube (n : ) : HomogeneousCubic ((PureU1Charges n).Charges) :=
(accCubeTriLinSymm).toCubic
lemma accCube_explicit (n : ) (S : (PureU1Charges n).Charges) :
accCube n S = ∑ i : Fin n, S i ^ 3:= by
rw [accCube, TriLinearSymm.toCubic]
@ -177,5 +174,4 @@ lemma sum_of_anomaly_free_linear {n : } (f : Fin k → (PureU1 n).LinSols) (j
erw [← hlt]
simp
end PureU1