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 #
Polynomial.logMahlerMeasure p: the logarithmic Mahler measure of a polynomialpdefined as(2 * π)⁻¹ * ∫ x ∈ (0, 2 * π), log ‖p (e ^ (i * x))‖.Polynomial.mahlerMeasure p: the (exponential) Mahler measure of a polynomialp, which is equal toe ^ p.logMahlerMeasureifpis nonzero, and0otherwise.
Main results #
Polynomial.mahlerMeasure_mul: the Mahler measure of the product of two polynomials is the product of their Mahler measures.mahlerMeasure_eq_leadingCoeff_mul_prod_roots: 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.
The logarithmic Mahler measure of a polynomial p defined as
(2 * π)⁻¹ * ∫ x ∈ (0, 2 * π), log ‖p (e ^ (i * x))‖
Equations
- p.logMahlerMeasure = Real.circleAverage (fun (x : ℂ) => Real.log ‖Polynomial.eval x p‖) 0 1
Instances For
The Mahler measure of a polynomial p defined as e ^ (logMahlerMeasure p) if p is nonzero
and 0 otherwise
Equations
- p.mahlerMeasure = if p ≠ 0 then Real.exp p.logMahlerMeasure else 0
Instances For
The Mahler measure of the product of two polynomials is the product of their Mahler measures
Alias of Polynomial.logMahlerMeasure_mul_eq_add_logMahlerMeasure.
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.