nevanlinna/Nevanlinna/holomorphic_zero.lean

37 lines
875 B
Plaintext
Raw Normal View History

2024-08-16 09:20:42 +02:00
import Mathlib.Analysis.Analytic.IsolatedZeros
2024-08-16 07:13:38 +02:00
import Nevanlinna.holomorphic
2024-08-16 09:20:42 +02:00
noncomputable def zeroDivisor
(f : ) :
:= by
intro z
if hf : AnalyticAt f z then
exact hf.order.toNat
else
exact 0
theorem discreteZeros
{f : } :
DiscreteTopology (Function.support (zeroDivisor f)) := by
sorry
theorem zeroDivisor_finiteOnCompact
2024-08-16 07:13:38 +02:00
{f : }
2024-08-16 09:20:42 +02:00
{s : Set }
(hs : IsCompact s) :
Set.Finite (s ∩ Function.support (zeroDivisor f)) := by
sorry
theorem eliminatingZeros
{f : }
{z₀ : }
2024-08-16 07:13:38 +02:00
{R : }
2024-08-16 09:20:42 +02:00
(h₁f : ∀ z ∈ Metric.ball z₀ R, HolomorphicAt f z)
(h₂f : ∃ z ∈ Metric.ball z₀ R, f z ≠ 0) :
∃ F : , ∀ z ∈ Metric.ball z₀ R, (HolomorphicAt F z) ∧ (f z = (F z) * ∏ᶠ a ∈ Metric.ball z₀ R, (z - a) ^ (zeroDivisor f a) ) := by
2024-08-16 07:13:38 +02:00
sorry