The Positive Part of the Logarithm #
This file defines the function Real.posLog = r ↦ max 0 (log r)
and introduces the notation
log⁺
. For a finite length-n
sequence f i
of reals, it establishes the following standard
estimates.
theorem posLog_prod : log⁺ (∏ i, f i) ≤ ∑ i, log⁺ (f i)
theorem posLog_sum : log⁺ (∑ i, f i) ≤ log n + ∑ i, log⁺ (f i)
Definition, Notation and Reformulations #
Notation log⁺
for the positive part of the logarithm.
Equations
- Real.«termLog⁺» = Lean.ParserDescr.node `Real.«termLog⁺» 1024 (Lean.ParserDescr.symbol "log⁺")
Instances For
Elementary Properties #
The function log⁺
is monotone on the positive axis.
Estimates for Products #
Estimate for log⁺
of a product. See Real.posLog_prod
for a variant involving
multiple factors.
Estimate for log⁺
of a product. See Real.posLog_mul
for a variant with
only two factors.