nevanlinna/Nevanlinna/firstMain.lean

184 lines
4.2 KiB
Plaintext
Raw Normal View History

2024-12-05 16:53:48 +01:00
import Mathlib.MeasureTheory.Integral.CircleIntegral
2024-12-05 13:51:00 +01:00
import Nevanlinna.divisor
2024-12-05 16:53:48 +01:00
import Nevanlinna.stronglyMeromorphicOn
import Nevanlinna.meromorphicOn_divisor
2024-12-19 16:10:51 +01:00
import Nevanlinna.meromorphicOn_integrability
2024-09-13 09:21:57 +02:00
open Real
2024-12-05 16:53:48 +01:00
-- Lang p. 164
2024-12-09 19:58:56 +01:00
theorem MeromorphicOn.restrict
{f : }
(h₁f : MeromorphicOn f )
(r : ) :
MeromorphicOn f (Metric.closedBall 0 r) := by
exact fun x a => h₁f x trivial
2024-12-20 08:16:22 +01:00
theorem MeromorphicOn.restrict_inv
{f : }
(h₁f : MeromorphicOn f )
(r : ) :
h₁f.inv.restrict r = (h₁f.restrict r).inv := by
funext x
simp
2024-12-05 16:53:48 +01:00
noncomputable def MeromorphicOn.N_zero
{f : }
2024-12-09 19:58:56 +01:00
(hf : MeromorphicOn f ) :
2024-12-05 16:53:48 +01:00
:=
2024-12-09 19:58:56 +01:00
fun r ↦ ∑ᶠ z, (max 0 ((hf.restrict r).divisor z)) * log (r * ‖z‖⁻¹)
2024-12-05 16:53:48 +01:00
noncomputable def MeromorphicOn.N_infty
{f : }
2024-12-09 19:58:56 +01:00
(hf : MeromorphicOn f ) :
2024-12-05 16:53:48 +01:00
:=
2024-12-09 19:58:56 +01:00
fun r ↦ ∑ᶠ z, (max 0 (-((hf.restrict r).divisor z))) * log (r * ‖z‖⁻¹)
2024-12-05 16:53:48 +01:00
2024-12-20 08:16:22 +01:00
theorem Nevanlinna_counting₀
{f : }
(hf : MeromorphicOn f ) :
hf.inv.N_infty = hf.N_zero := by
funext r
unfold MeromorphicOn.N_zero MeromorphicOn.N_infty
let A := (hf.restrict r).divisor.finiteSupport (isCompact_closedBall 0 r)
repeat
rw [finsum_eq_sum_of_support_subset (s := A.toFinset)]
apply Finset.sum_congr rfl
intro x hx
congr
rw [hf.restrict_inv r]
rw [MeromorphicOn.divisor_inv]
simp
--
exact fun x a => hf x trivial
--
intro x
contrapose
simp
intro hx
rw [hx]
tauto
--
intro x
contrapose
simp
intro hx h₁x
rw [hf.restrict_inv r] at h₁x
have hh : MeromorphicOn f (Metric.closedBall 0 r) := hf.restrict r
rw [hh.divisor_inv] at h₁x
simp at h₁x
rw [hx] at h₁x
tauto
2024-12-05 16:53:48 +01:00
theorem Nevanlinna_counting
{f : }
2024-12-09 19:58:56 +01:00
(hf : MeromorphicOn f ) :
hf.N_zero - hf.N_infty = fun r ↦ ∑ᶠ z, ((hf.restrict r).divisor z) * log (r * ‖z‖⁻¹) := by
2024-12-09 16:00:26 +01:00
funext r
simp only [Pi.sub_apply]
2024-12-09 19:58:56 +01:00
unfold MeromorphicOn.N_zero MeromorphicOn.N_infty
let A := (hf.restrict r).divisor.finiteSupport (isCompact_closedBall 0 r)
repeat
rw [finsum_eq_sum_of_support_subset (s := A.toFinset)]
rw [← Finset.sum_sub_distrib]
simp_rw [← sub_mul]
congr
funext x
congr
by_cases h : 0 ≤ (hf.restrict r).divisor x
· simp [h]
· have h' : 0 ≤ -((hf.restrict r).divisor x) := by
simp at h
apply Int.le_neg_of_le_neg
simp
exact Int.le_of_lt h
simp at h
simp [h']
linarith
--
repeat
intro x
contrapose
simp
intro hx
rw [hx]
tauto
2024-12-05 16:53:48 +01:00
2024-09-14 08:38:04 +02:00
2024-12-05 16:53:48 +01:00
--
noncomputable def MeromorphicOn.m_infty
{f : }
2024-12-09 19:58:56 +01:00
(_ : MeromorphicOn f ) :
2024-12-05 16:53:48 +01:00
:=
fun r ↦ (2 * π)⁻¹ * ∫ x in (0)..(2 * π), logpos ‖f (circleMap 0 r x)‖
2024-12-19 16:10:51 +01:00
2024-12-05 16:53:48 +01:00
theorem Nevanlinna_proximity
{f : }
{r : }
(h₁f : MeromorphicOn f ) :
(2 * π)⁻¹ * ∫ x in (0)..(2 * π), log ‖f (circleMap 0 r x)‖ = (h₁f.m_infty r) - (h₁f.inv.m_infty r) := by
2024-12-19 16:10:51 +01:00
2024-12-05 16:53:48 +01:00
unfold MeromorphicOn.m_infty
rw [← mul_sub]; congr
rw [← intervalIntegral.integral_sub]; congr
funext x
simp_rw [loglogpos]; congr
exact Eq.symm (IsAbsoluteValue.abv_inv Norm.norm (f (circleMap 0 r x)))
--
2024-12-19 21:24:13 +01:00
apply MeromorphicOn.integrable_logpos_abs_f
2024-12-20 08:16:22 +01:00
intro z hx
exact h₁f z trivial
--
apply MeromorphicOn.integrable_logpos_abs_f
exact MeromorphicOn.inv_iff.mpr fun x a => h₁f x trivial
2024-12-19 16:10:51 +01:00
2024-12-19 21:24:13 +01:00
2024-12-05 16:53:48 +01:00
noncomputable def MeromorphicOn.T_infty
{f : }
(hf : MeromorphicOn f ) :
2024-12-05 13:51:00 +01:00
:=
2024-12-05 16:53:48 +01:00
hf.m_infty + hf.N_infty
2024-12-20 08:16:22 +01:00
2024-12-05 16:53:48 +01:00
theorem Nevanlinna_firstMain₁
{f : }
(h₁f : MeromorphicOn f )
(h₂f : StronglyMeromorphicAt f 0)
(h₃f : f 0 ≠ 0) :
(fun r ↦ log ‖f 0‖) + h₁f.inv.T_infty = h₁f.T_infty := by
2024-12-20 08:16:22 +01:00
rw [add_eq_of_eq_sub]
unfold MeromorphicOn.T_infty
have {A B C D : } : A + B - (C + D) = A - C + (B - D) := by
ring
rw [this]
clear this
2024-12-05 16:53:48 +01:00
funext r
simp
2024-12-20 08:16:22 +01:00
rw [← Nevanlinna_proximity h₁f]
2024-12-05 16:53:48 +01:00
unfold MeromorphicOn.N_infty
unfold MeromorphicOn.m_infty
simp
sorry
theorem Nevanlinna_firstMain₂
{f : }
{a : }
{r : }
(h₁f : MeromorphicOn f ) :
|(h₁f.T_infty r) - ((h₁f.sub (MeromorphicOn.const a)).T_infty r)| ≤ logpos ‖a‖ + log 2 := by
sorry