Skip to content

Commit

Permalink
fix:NumberTheory.LegendreSymbol.GaussSum fix porting note (#5525)
Browse files Browse the repository at this point in the history
Forgot to write a porting note
  • Loading branch information
xroblot committed Jun 27, 2023
1 parent c660824 commit 8f691fc
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/NumberTheory/LegendreSymbol/GaussSum.lean
Expand Up @@ -163,7 +163,7 @@ theorem gaussSum_frob (χ : MulChar R R') (ψ : AddChar R R') :
/-- For a quadratic character `χ` and when the characteristic `p` of the target ring
is a unit in the source ring, the `p`th power of the Gauss sum of`χ` and `ψ` is
`χ p` times the original Gauss sum. -/
-- Porting note: TODO
-- Porting note: Added `nonrec` to avoid error `failed to prove termination`
nonrec theorem MulChar.IsQuadratic.gaussSum_frob (hp : IsUnit (p : R)) {χ : MulChar R R'}
(hχ : IsQuadratic χ) (ψ : AddChar R R') : gaussSum χ ψ ^ p = χ p * gaussSum χ ψ := by
rw [gaussSum_frob, pow_mulShift, hχ.pow_char p, ← gaussSum_mulShift χ ψ hp.unit, ← mul_assoc,
Expand Down

0 comments on commit 8f691fc

Please sign in to comment.