Documentation

Mathlib.Analysis.Complex.ValueDistribution.ProximityFunction

The Proximity Function of Value Distribution Theory #

This file defines the "proximity function" attached to a meromorphic function defined on the complex plane. Also known as the Nevanlinna Proximity Function, this is one of the three main functions used in Value Distribution Theory.

The proximity function is a logarithmically weighted measure quantifying how well a meromorphic function f approximates the constant function a on the circle of radius R in the complex plane. The definition ensures that large values correspond to good approximation.

See SectionVI.2 of Lang, Introduction to Complex Hyperbolic Spaces or Section1.1 of Noguchi-Winkelmann, Nevanlinna Theory in Several Complex Variables and Diophantine Approximation for a detailed discussion.

noncomputable def ValueDistribution.proximity {E : Type u_1} [NormedAddCommGroup E] (f : E) (a : WithTop E) :

The Proximity Function of Value Distribution Theory

If f : ℂ → E is meromorphic and a : WithTop E is any value, the proximity function is a logarithmically weighted measure quantifying how well a meromorphic function f approximates the constant function a on the circle of radius R in the complex plane. In the special case where a = ⊤, it quantifies how well f approximates infinity.

Equations
Instances For
    theorem ValueDistribution.proximity_coe {E : Type u_1} [NormedAddCommGroup E] {f : E} {a₀ : E} :
    proximity f a₀ = Real.circleAverage (fun (x : ) => f x - a₀⁻¹.posLog) 0

    Expand the definition of proximity f a₀ in case where a₀ is finite.

    Expand the definition of proximity f a₀ in case where a₀ is zero.

    For complex-valued functions, expand the definition of proximity f a₀ in case where a₀ is zero. This is a simple variant of proximity_zero defined above.

    Expand the definition of proximity f a in case where a₀ = ⊤.

    Elementary Properties of the Counting Function #

    theorem ValueDistribution.proximity_coe_eq_proximity_sub_const_zero {E : Type u_1} [NormedAddCommGroup E] {f : E} {a₀ : E} :
    proximity f a₀ = proximity (f - fun (x : ) => a₀) 0

    For finite values a₀, the proximity function proximity f a₀ equals the proximity function for the value zero of the shifted function f - a₀.

    For complex-valued f, establish a simple relation between the proximity functions of f and of f⁻¹.