Documentation

Mathlib.Analysis.Polynomial.MahlerMeasure

Mahler measure of complex polynomials #

In this file we define the Mahler measure of a polynomial over ℂ[X] and prove some basic properties.

Main definitions #

Main results #

The logarithmic Mahler measure of a polynomial p defined as (2 * π)⁻¹ * ∫ x ∈ (0, 2 * π), log ‖p (e ^ (i * x))‖

Equations
Instances For
    noncomputable def Polynomial.mahlerMeasure (p : Polynomial ) :

    The Mahler measure of a polynomial p defined as e ^ (logMahlerMeasure p) if p is nonzero and 0 otherwise

    Equations
    Instances For

      The Mahler measure of the product of two polynomials is the product of their Mahler measures

      @[deprecated Polynomial.logMahlerMeasure_mul_eq_add_logMahlerMeasure (since := "2025-11-17")]

      Alias of Polynomial.logMahlerMeasure_mul_eq_add_logMahlerMeasure.

      @[simp]

      The logarithmic Mahler measure of X - C z is the log⁺ of the absolute value of z.

      @[simp]

      The Mahler measure of X - C z equals max 1 ‖z‖.

      @[simp]

      The logarithmic Mahler measure of a polynomial is the log of the absolute value of its leading coefficient plus the sum of the logs of the absolute values of its roots lying outside the unit disk.

      The Mahler measure of a polynomial is the absolute value of its leading coefficient times the product of the absolute values of its roots lying outside the unit disk.

      Estimates for the Mahler measure #

      The Mahler measure of a polynomial is bounded above by the sum of the norms of its coefficients.