Documentation

Mathlib.Analysis.SpecialFunctions.Log.NegMulLog

The function x ↦ - x * log x #

The purpose of this file is to record basic analytic properties of the function x ↦ - x * log x, which is notably used in the theory of Shannon entropy.

Main definitions #

theorem Real.deriv_mul_log {x : } (hx : x 0) :
deriv (fun (x : ) => x * Real.log x) x = Real.log x + 1
theorem Real.hasDerivAt_mul_log {x : } (hx : x 0) :
HasDerivAt (fun (x : ) => x * Real.log x) (Real.log x + 1) x
theorem Real.deriv2_mul_log {x : } (hx : x 0) :
deriv^[2] (fun (x : ) => x * Real.log x) x = x⁻¹
theorem Real.mul_log_nonneg {x : } (hx : 1 x) :
0 x * Real.log x
theorem Real.mul_log_nonpos {x : } (hx₀ : 0 x) (hx₁ : x 1) :
x * Real.log x 0
noncomputable def Real.negMulLog (x : ) :

The function x ↦ - x * log x from to .

Equations
Instances For
    theorem Real.negMulLog_nonneg {x : } (h1 : 0 x) (h2 : x 1) :
    theorem Real.deriv2_negMulLog {x : } (hx : x 0) :