Skip to content

Commit

Permalink
ZetaInvBnd work
Browse files Browse the repository at this point in the history
  • Loading branch information
AlexKontorovich committed May 6, 2024
1 parent 0daa772 commit 43455aa
Showing 1 changed file with 8 additions and 4 deletions.
12 changes: 8 additions & 4 deletions PrimeNumberTheoremAnd/ZetaBounds.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1730,11 +1730,15 @@ lemma ZetaInvBnd :
(hσ : σ ∈ Ico (1 - A / (Real.log |t|) ^ 9) 1),
1 / ‖ζ (σ + t * I)‖ ≤ C * (Real.log |t|) ^ 7 := by
obtain ⟨A', hA', C', hC', h'⟩ := Zeta_diff_Bnd
let A := min A' <| (1 / 16 : ℝ)
obtain ⟨C₂, C₂pos, hC'⟩ := ZetaInvBound2
let A := min A' <| (1 / 2 : ℝ) * (C' / 2 * C₂) ^ 4
have Apos : 0 < A := by have := hA'.1; positivity
let C := C'
have Cpos : 0 < C := by positivity
refine ⟨A, ⟨Apos, by norm_num [A]⟩ , C, Cpos, ?_⟩
have A_le_A' : A ≤ A' := by simp [A]
let C := C' * A ^ (3 / 4 : ℝ) - 2 * A * C₂
have Cpos : 0 < C := by
apply sub_pos.mpr
sorry
refine ⟨A, ⟨Apos, by linarith [hA'.2]⟩ , C, Cpos, ?_⟩
intro σ t t_gt hσ
have logt_gt_one := logt_gt_one t_gt
have σ_ge : 1 - A / |t|.log ≤ σ := by
Expand Down

0 comments on commit 43455aa

Please sign in to comment.