Representation of log⁺
as a Circle Average #
If a
is any complex number, circleAverage_log_norm_sub_const_eq_posLog
represents log⁺ a
as
the circle average of log ‖· - a‖
over the unit circle.
Circle Integrability #
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
. #
Computing circleAverage (log ‖· - a‖) 0 1
in case where ‖a‖ = 1
. #
Computing circleAverage (log ‖· - a‖) 0 1
in case where 1 < ‖a‖
. #
Presentation of log⁺
in Terms of Circle Averages #
Generalization of circleAverage_log_norm_sub_const_eq_posLog
: The
circleAverage (log ‖· - a‖) c R
equals log R + log⁺ (|R|⁻¹ * ‖c - a‖)
.
theorem
circleAverage_log_norm_sub_const_of_mem_closedBall
{a c : ℂ}
{R : ℝ}
(hu : a ∈ Metric.closedBall c |R|)
:
Trivial corollary of
circleAverage_log_norm_sub_const_eq_log_radius_add_posLog
: If u : ℂ
lies within the closed ball
with center c
and radius R
, then the circle average
circleAverage (log ‖· - u‖) c R
equals log R
.