nevanlinna/Nevanlinna/meromorphicOn_integrability.lean

70 lines
1.8 KiB
Plaintext
Raw Normal View History

2024-12-11 12:36:44 +01:00
import Mathlib.Analysis.Analytic.Meromorphic
import Nevanlinna.analyticAt
import Nevanlinna.divisor
import Nevanlinna.meromorphicAt
import Nevanlinna.meromorphicOn_divisor
import Nevanlinna.stronglyMeromorphicOn
import Nevanlinna.mathlibAddOn
import Mathlib.MeasureTheory.Integral.CircleIntegral
open scoped Interval Topology
open Real Filter MeasureTheory intervalIntegral
2024-12-13 07:58:40 +01:00
lemma b
(S U : Set )
(hS : S ∈ Filter.codiscreteWithin U) :
DiscreteTopology ((S Uᶜ)ᶜ : Set ) := by
2024-12-12 13:49:33 +01:00
rw [mem_codiscreteWithin] at hS
simp at hS
2024-12-13 07:58:40 +01:00
have : (U \ S)ᶜ = S Uᶜ := by
ext z
simp
tauto
2024-12-12 13:49:33 +01:00
rw [discreteTopology_subtype_iff]
intro x hx
rw [← mem_iff_inf_principal_compl]
2024-12-13 07:58:40 +01:00
simp at hx
let A := hS x hx.2
rw [← this]
assumption
lemma c
(S U : Set )
(hS : S ∈ Filter.codiscreteWithin U) :
Countable ((S Uᶜ)ᶜ : Set ) := by
let A := b S U hS
apply TopologicalSpace.separableSpace_iff_countable.1
exact TopologicalSpace.SecondCountableTopology.to_separableSpace
2024-12-12 13:49:33 +01:00
2024-12-11 12:36:44 +01:00
theorem integrability_congr_changeDiscrete
{f₁ f₂ : }
2024-12-13 07:58:40 +01:00
{U : Set }
2024-12-11 12:36:44 +01:00
{r : }
2024-12-13 07:58:40 +01:00
(hf : f₁ =ᶠ[Filter.codiscreteWithin U] f₂) :
2024-12-11 12:36:44 +01:00
IntervalIntegrable (f₁ ∘ (circleMap 0 r)) MeasureTheory.volume 0 (2 * π) → IntervalIntegrable (f₂ ∘ (circleMap 0 r)) MeasureTheory.volume 0 (2 * π) := by
intro hf₁
apply IntervalIntegrable.congr hf₁
rw [Filter.eventuallyEq_iff_exists_mem]
2024-12-13 07:58:40 +01:00
use (circleMap 0 r)⁻¹' ({z | f₁ z = f₂ z} ∩ U)
2024-12-11 12:36:44 +01:00
constructor
· apply Set.Countable.measure_zero
2024-12-13 07:58:40 +01:00
have : (circleMap 0 r ⁻¹' ({z | f₁ z = f₂ z} ∩ U))ᶜ = (circleMap 0 r ⁻¹' ({z | f₁ z = f₂ z} ∩ U)ᶜ) := by
2024-12-11 12:36:44 +01:00
exact rfl
rw [this]
apply Set.Countable.preimage_circleMap
2024-12-13 07:58:40 +01:00
apply c
2024-12-11 12:36:44 +01:00
sorry
sorry
2024-12-13 07:58:40 +01:00
· intro x hx
simp at hx
simp
exact hx.1