Skip to content

Commit

Permalink
chore(NumberTheory/ModularForms/JacobiTheta): simplify proof of isBig…
Browse files Browse the repository at this point in the history
…O_atTop_F_int_zero_sub (#19879)

* `have ha' : (a : UnitAddCircle) = 0 ↔ a = 0` can be directly proved by `AddCircle.coe_eq_zero_iff_of_mem_Ico ha`.
* That makes the proof small enough that it makes sense to inline it at its use in `simp_rw`.

This simplification was found by [`tryAtEachStep`](https://github.com/dwrensha/tryAtEachStep).
  • Loading branch information
dwrensha committed Dec 11, 2024
1 parent f7bc890 commit d840f50
Showing 1 changed file with 1 addition and 5 deletions.
6 changes: 1 addition & 5 deletions Mathlib/NumberTheory/ModularForms/JacobiTheta/Bounds.lean
Original file line number Diff line number Diff line change
Expand Up @@ -249,11 +249,7 @@ lemma isBigO_atTop_F_int_zero_sub (a : UnitAddCircle) : ∃ p, 0 < p ∧
obtain ⟨a, ha, rfl⟩ := a.eq_coe_Ico
obtain ⟨p, hp, hp'⟩ := isBigO_atTop_F_nat_zero_sub ha.1
obtain ⟨q, hq, hq'⟩ := isBigO_atTop_F_nat_zero_sub (sub_nonneg.mpr ha.2.le)
have ha' : (a : UnitAddCircle) = 0 ↔ a = 0 := by
rw [← AddCircle.coe_eq_coe_iff_of_mem_Ico (hp := ⟨zero_lt_one' ℝ⟩), QuotientAddGroup.mk_zero]
· rw [zero_add]; exact ha
· simp
simp_rw [ha']
simp_rw [AddCircle.coe_eq_zero_iff_of_mem_Ico ha]
simp_rw [eq_false_intro (by linarith [ha.2] : 1 - a ≠ 0), if_false, sub_zero] at hq'
refine ⟨_, lt_min hp hq, ?_⟩
have : (fun t ↦ F_int 0 a t - (if a = 0 then 1 else 0)) =ᶠ[atTop]
Expand Down

0 comments on commit d840f50

Please sign in to comment.