Documentation

Mathlib.Analysis.SpecialFunctions.Integrals.PosLogEqCircleAverage

Representation of log⁺ as a Circle Average #

If a is any complex number of norm one, then log ‖· - a‖ is circle integrable over every circle in the complex plane, and the circle average circleAverage (log ‖· - a‖) 0 1 vanishes.

TODO: As soon as the mean value theorem for harmonic functions becomes available, extend this result to arbitrary complex numbers a, showing that the circle average equals the positive part of the logarithm, circleAverage (log ‖· - a‖) 0 1 = = log⁺ ‖a‖. This result, in turn, is a major ingredient in the proof of Jensen's formula in complex analysis.

Circle Integrability #

theorem circleIntegrable_log_norm_sub_const {a c : } (r : ) :
CircleIntegrable (fun (x : ) => Real.log x - a) c r

If a is any complex number, the function (log ‖· - a‖) is circle integrable over every circle.

Computing circleAverage (log ‖· - a‖) 0 1 in case where ‖a‖ = 1. #

@[simp]
theorem circleAverage_log_norm_sub_const₁ {a : } (h : a = 1) :
Real.circleAverage (fun (x : ) => Real.log x - a) 0 1 = 0

If a : ℂ has norm one, then the circle average circleAverage (log ‖· - a‖) 0 1 vanishes.