This commit is contained in:
Stefan Kebekus 2024-11-07 12:08:52 +01:00
parent e843786097
commit dfc67cec4a
2 changed files with 26 additions and 3 deletions

View File

@ -0,0 +1,23 @@
import Mathlib.Analysis.Analytic.Meromorphic
import Nevanlinna.analyticAt
import Nevanlinna.divisor
import Nevanlinna.meromorphicAt
import Nevanlinna.meromorphicOn_divisor
import Nevanlinna.stronglyMeromorphicOn
open scoped Interval Topology
open Real Filter MeasureTheory intervalIntegral
theorem MeromorphicOn.decompose
{f : }
{U : Set }
(h₁U : IsConnected U)
(h₂U : IsCompact U)
(h₁f : MeromorphicOn f U)
(h₂f : ∃ z₀ ∈ U, f z₀ ≠ 0) :
∃ g : , (AnalyticOnNhd g U)
∧ (∀ z ∈ U, g z ≠ 0)
∧ (Set.EqOn h₁f.makeStronglyMeromorphicOn (fun z ↦ ∏ᶠ p ∈ h₁f.divisor.support, (z-p) ) U) := by
sorry

View File

@ -155,7 +155,7 @@ lemma m₂
apply eventually_nhdsWithin_of_forall apply eventually_nhdsWithin_of_forall
exact fun x a => m₁ hf x a exact fun x a => m₁ hf x a
/-
lemma Mnhds lemma Mnhds
{f g : } {f g : }
{z₀ : } {z₀ : }
@ -172,7 +172,7 @@ lemma Mnhds
· simp at h₂y · simp at h₂y
rwa [h₂y] rwa [h₂y]
· exact h₂t · exact h₂t
-/
theorem localIdentity theorem localIdentity
{f g : } {f g : }
@ -262,7 +262,7 @@ theorem makeStronglyMeromorphic_id
· rw [hz] · rw [hz]
unfold MeromorphicAt.makeStronglyMeromorphicAt unfold MeromorphicAt.makeStronglyMeromorphicAt
simp simp
let h₀f := hf have h₀f := hf
rcases hf with h₁f|h₁f rcases hf with h₁f|h₁f
· have A : f =ᶠ[𝓝[≠] z₀] 0 := by · have A : f =ᶠ[𝓝[≠] z₀] 0 := by
apply Filter.EventuallyEq.filter_mono h₁f apply Filter.EventuallyEq.filter_mono h₁f