nevanlinna/Nevanlinna/divisor.lean

23 lines
578 B
Plaintext
Raw Normal View History

2024-09-30 14:12:33 +02:00
import Mathlib.Analysis.SpecialFunctions.Integrals
import Mathlib.Analysis.SpecialFunctions.Log.NegMulLog
import Mathlib.Analysis.Convex.SpecificFunctions.Deriv
2024-09-14 08:38:04 +02:00
import Nevanlinna.analyticAt
2024-10-07 07:56:42 +02:00
open Interval Topology
2024-09-30 14:12:33 +02:00
open Real Filter MeasureTheory intervalIntegral
2024-10-07 07:56:42 +02:00
structure Divisor
(U : Set )
where
2024-09-14 08:38:04 +02:00
toFun :
2024-10-07 07:56:42 +02:00
supportInU : toFun.support ⊆ U
locallyFiniteInU : ∀ x ∈ U, ∃ N ∈ 𝓝 x, (N ∩ toFun.support).Finite
2024-09-17 11:03:44 +02:00
2024-10-07 07:56:42 +02:00
instance
(U : Set ) :
CoeFun (Divisor U) (fun _ ↦ ) where
coe := Divisor.toFun
2024-09-17 11:03:44 +02:00
2024-10-07 07:56:42 +02:00
attribute [coe] Divisor.toFun