Documentation

Mathlib.Data.Real.ConjExponents

Real conjugate exponents #

This file defines conjugate exponents in and ℝ≥0. Real numbers p and q are conjugate if they are both greater than 1 and satisfy p⁻¹ + q⁻¹ = 1. This property shows up often in analysis, especially when dealing with L^p spaces.

Main declarations #

TODO #

structure Real.IsConjExponent (p q : ) :

Two real exponents p, q are conjugate if they are > 1 and satisfy the equality 1/p + 1/q = 1. This condition shows up in many theorems in analysis, notably related to L^p norms.

Instances For

    The conjugate exponent of p is q = p/(p-1), so that 1/p + 1/q = 1.

    Equations
    Instances For
      theorem Real.IsConjExponent.pos {p q : } (h : p.IsConjExponent q) :
      0 < p
      theorem Real.IsConjExponent.conj_eq {p q : } (h : p.IsConjExponent q) :
      q = p / (p - 1)
      theorem Real.IsConjExponent.sub_one_mul_conj {p q : } (h : p.IsConjExponent q) :
      (p - 1) * q = p
      theorem Real.IsConjExponent.mul_eq_add {p q : } (h : p.IsConjExponent q) :
      p * q = p + q
      theorem Real.IsConjExponent.inv_inv {a b : } (ha : 0 < a) (hb : 0 < b) (hab : a + b = 1) :
      theorem Real.IsConjExponent.inv_one_sub_inv {a : } (ha₀ : 0 < a) (ha₁ : a < 1) :
      theorem Real.IsConjExponent.one_sub_inv_inv {a : } (ha₀ : 0 < a) (ha₁ : a < 1) :
      theorem Real.isConjExponent_iff_eq_conjExponent {p q : } (hp : 1 < p) :
      p.IsConjExponent q q = p / (p - 1)
      theorem Real.isConjExponent_one_div {a b : } (ha : 0 < a) (hb : 0 < b) (hab : a + b = 1) :
      (1 / a).IsConjExponent (1 / b)
      structure NNReal.IsConjExponent (p q : NNReal) :

      Two nonnegative real exponents p, q are conjugate if they are > 1 and satisfy the equality 1/p + 1/q = 1. This condition shows up in many theorems in analysis, notably related to L^p norms.

      Instances For
        noncomputable def NNReal.conjExponent (p : NNReal) :

        The conjugate exponent of p is q = p/(p-1), so that 1/p + 1/q = 1.

        Equations
        Instances For
          theorem NNReal.IsConjExponent.coe {p q : NNReal} :
          p.IsConjExponent q(↑p).IsConjExponent q

          Alias of the reverse direction of NNReal.isConjExponent_coe.

          theorem NNReal.IsConjExponent.conj_eq {p q : NNReal} (h : p.IsConjExponent q) :
          q = p / (p - 1)
          theorem NNReal.IsConjExponent.inv_inv {a b : NNReal} (ha : a 0) (hb : b 0) (hab : a + b = 1) :
          theorem NNReal.IsConjExponent.inv_one_sub_inv {a : NNReal} (ha₀ : a 0) (ha₁ : a < 1) :
          theorem NNReal.IsConjExponent.one_sub_inv_inv {a : NNReal} (ha₀ : a 0) (ha₁ : a < 1) :

          Two extended nonnegative real exponents p, q are conjugate and satisfy the equality 1/p + 1/q = 1. This condition shows up in many theorems in analysis, notably related to L^p norms. Note that we permit one of the exponents to be and the other 1.

          Instances For
            noncomputable def ENNReal.conjExponent (p : ENNReal) :

            The conjugate exponent of p is q = 1 + (p - 1)⁻¹, so that 1/p + 1/q = 1.

            Equations
            Instances For
              theorem ENNReal.coe_conjExponent {p : NNReal} (hp : 1 < p) :

              Alias of the reverse direction of ENNReal.isConjExponent_coe.