Skip to content

Commit

Permalink
chore: add try (#18344)
Browse files Browse the repository at this point in the history
It's a Lean bug that `try` was not necessary here. (Will be fixed in lean4#5863.)
  • Loading branch information
kmill committed Oct 29, 2024
1 parent 3e82c09 commit 5a79791
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/NumberTheory/LSeries/MellinEqDirichlet.lean
Original file line number Diff line number Diff line change
Expand Up @@ -92,7 +92,7 @@ lemma hasSum_mellin_pi_mul₀ {a : ι → ℂ} {p : ι → ℝ} {F : ℝ → ℂ
let a' i := if p i = 0 then 0 else a i
have hp' i : a' i = 00 < p i := by
simp only [a']
split_ifs with h <;> tauto
split_ifs with h <;> try tauto
exact Or.inr (lt_of_le_of_ne (hp i) (Ne.symm h))
have (i t) : (if p i = 0 then 0 else a i * rexp (-π * p i * t)) =
a' i * rexp (-π * p i * t) := by
Expand Down

0 comments on commit 5a79791

Please sign in to comment.