nevanlinna/Nevanlinna/firstMain.lean

18 lines
534 B
Plaintext
Raw Normal View History

2024-09-13 09:21:57 +02:00
import Nevanlinna.holomorphic_JensenFormula
open Real
variable {f : }
variable {h₁f : AnalyticOn f }
variable {h₂f : f 0 ≠ 0}
noncomputable def unintegratedCounting : := by
intro r
let A := h₁f.mono (by tauto : Metric.closedBall (0 : ) r ⊆ )
exact ∑ᶠ z, (A.order z).toNat
noncomputable def integratedCounting : := by
intro r
-- Issue here: for s on the boundary of the ball, zero comes out.
exact ∑ᶠ s, (h₁f.order s).toNat * log (r * ‖s.1‖⁻¹)