Documentation

FormalConjectures.Wikipedia.PierceBirkhoff

Pierce–Birkhoff conjecture #

Reference: Wikipedia

The Pierce-Birkhoff conjecture asserts that any piecewise-polynomial function can be expressed as a maximum of finite minima of finite collections of polynomials. It was first stated in 1956 by Garrett Birkhoff and Richard S. Pierce, though the modern rigorous formulation is due to Melvin Henriksen and John R. Isbell.

The conjecture has been proved for n = 1 and n = 2 by Louis Mahé.

A set is semi-algebraic in ℝⁿ if it can be described by a finite union of sets defined by multivariate polynomial equations and inequalities.

Equations
  • One or more equations did not get rendered due to their size.
Instances For

    A set is semi-algebraic in if it can be described by a finite boolean combination of polynomial equations and inequalities.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For

      A function f : ℝⁿ → ℝ is piecewise polynomial if there exists a finite covering of ℝⁿ by closed semi-algebraic sets such that the restriction of f to each set in the covering is polynomial.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For

        A function f : ℝ → ℝ is piecewise polynomial if there exists a finite covering of by closed semi-algebraic sets such that the restriction of f to each set in the covering is polynomial.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          theorem pierce_birkhoff_conjecture {n : } (f : EuclideanSpace (Fin n)) (hf : IsPiecewiseMvPolynomial f) :
          ∃ (ι : Type) (κ : Type) (g : ικMvPolynomial (Fin n) ), Finite ι Finite κ ∀ (x : EuclideanSpace (Fin n)), f x = ⨆ (i : ι), ⨅ (j : κ), (MvPolynomial.eval x) (g i j)

          The Pierce-Birkhoff conjecture states that for every real piecewise-polynomial function f : ℝⁿ → ℝ, there exists a finite set of polynomials gᵢⱼ ∈ ℝ[x₁, ..., xₙ] such that f = supᵢ infⱼ(gᵢⱼ).

          theorem pierce_birkhoff_conjecture_dim_one (f : ) (hf : IsPiecewisePolynomial f) :
          ∃ (ι : Type) (κ : Type) (g : ικPolynomial ), Finite ι Finite κ ∀ (x : ), f x = ⨆ (i : ι), ⨅ (j : κ), Polynomial.eval x (g i j)

          The Pierce-Birkhoff conjecture holds for n = 1. This was proved by Louis Mahé.

          theorem pierce_birkhoff_conjecture_dim_two (f : EuclideanSpace (Fin 2)) (hf : IsPiecewiseMvPolynomial f) :
          ∃ (ι : Type) (κ : Type) (g : ικMvPolynomial (Fin 2) ), Finite ι Finite κ ∀ (x : EuclideanSpace (Fin 2)), f x = ⨆ (i : ι), ⨅ (j : κ), (MvPolynomial.eval x) (g i j)

          The Pierce-Birkhoff conjecture holds for n = 2. This was proved by Louis Mahé.