Documentation

Frourio.Analysis.EntropyPackage

Entropy Functional Analysis Package #

This file provides the functional analytic framework for entropy functionals needed in the meta-variational principle.

Main API (Section 1-1 of plan2) #

Lower semicontinuity and chain rules (Section 1-2) #

Integrability conditions (Section 1-3) #

Implementation notes #

We use ℝ≥0∞ as the codomain for entropy functionals, converting to ℝ via toReal only when interfacing with PLFA/EVI frameworks.

For a probability measure μ, the relative entropy D(μ‖μ) equals zero. This is the key lemma from task 1-1 that highlights the self-entropy property.

theorem Frourio.relativeEntropy_lsc {X : Type u_1} [MeasurableSpace X] (μ : MeasureTheory.Measure X) [MeasureTheory.IsFiniteMeasure μ] (ρn : MeasureTheory.Measure X) (ρ : MeasureTheory.Measure X) (hacn : ∀ (n : ), (ρn n).AbsolutelyContinuous μ) (hac : ρ.AbsolutelyContinuous μ) (hfin_n : ∀ (n : ), MeasureTheory.IsFiniteMeasure (ρn n)) (hfin : MeasureTheory.IsFiniteMeasure ρ) (h_ae : ∀ᵐ (x : X) μ, Filter.Tendsto (fun (n : ) => ((ρn n).rnDeriv μ x).toReal) Filter.atTop (nhds (ρ.rnDeriv μ x).toReal)) :

Liminf-type lower semicontinuity of relative entropy under a.e. convergence of RN derivatives. If (ρₙ) and ρ are all absolutely continuous w.r.t. μ, and the RN derivatives (ρₙ.rnDeriv μ).toReal → (ρ.rnDeriv μ).toReal converge μ-a.e., then klDiv ρ μ ≤ liminf_n klDiv (ρₙ) μ holds by Fatou's lemma.

This is a key technical result for establishing LSC in the weak topology.

Relative entropy is non-negative

KL divergence equals zero iff measures are equal (for probability measures)

Core lemma: Additivity of log-likelihood ratios #

Under a multiplicative RN-derivative hypothesis, log-likelihood ratios add a.e. This is the key step towards the chain rule formula for KL divergences. It isolates the purely pointwise identity on log-likelihood ratios.

theorem Frourio.llr_add_of_rnDeriv_mul {X : Type u_1} [MeasurableSpace X] (μ ν ρ : MeasureTheory.Measure X) [MeasureTheory.SigmaFinite μ] [MeasureTheory.SigmaFinite ν] [MeasureTheory.SigmaFinite ρ] (hmul : ∀ᵐ (x : X) μ, (μ.rnDeriv ρ x).toReal = (μ.rnDeriv ν x).toReal * (ν.rnDeriv ρ x).toReal) (hpos1 : ∀ᵐ (x : X) μ, 0 < (μ.rnDeriv ν x).toReal) (hpos2 : ∀ᵐ (x : X) μ, 0 < (ν.rnDeriv ρ x).toReal) :
MeasureTheory.llr μ ρ =ᵐ[μ] fun (x : X) => MeasureTheory.llr μ ν x + MeasureTheory.llr ν ρ x

Chain rule for relative entropy (probability measure version with toReal).

For probability measures with μ ≪ ν ≪ ρ and appropriate integrability conditions, we have the chain rule: (klDiv μ ρ).toReal = (klDiv μ ν).toReal + ∫ llr ν ρ dμ

This is the concrete form needed for PLFA/EVI frameworks where we work with real values. The integrability assumptions h_int1 and h_int2 are explicit as required by plan2.

Section 1-3: Integrability conditions for chain rule #

These lemmas provide sufficient conditions to ensure the integrability assumptions required by the chain rule relativeEntropy_chain_rule_prob_toReal.

Transfer lemma: integrability of klFun composed with RN derivative implies integrability of llr. This is the main tool for verifying integrability conditions in the chain rule.

When the RN derivative is bounded, llr is integrable for finite measures. This provides a simple sufficient condition for integrability.

For probability measures with finite KL divergence, llr is integrable.

theorem Frourio.integrable_llr_of_uniform_bounds {X : Type u_1} [MeasurableSpace X] (μ ν : MeasureTheory.Measure X) [MeasureTheory.IsFiniteMeasure μ] [MeasureTheory.IsFiniteMeasure ν] (hμν : μ.AbsolutelyContinuous ν) (a b : ) (ha : 0 < a) (hb : a < b) (hbound : ∀ᵐ (x : X) ν, a (μ.rnDeriv ν x).toReal (μ.rnDeriv ν x).toReal b) :

When RN derivatives are uniformly bounded above and below, llr is integrable.

Data processing inequality: KL divergence decreases under stochastic maps

Entropy has compact sublevel sets (abstract statement)

Structure for entropy functional with functional analytic properties

Instances For

    Concrete entropy functional

    Equations
    Instances For
      theorem Frourio.entropy_displacement_convex {X : Type u_1} [MeasurableSpace X] [PseudoMetricSpace X] (μ : MeasureTheory.Measure X) [MeasureTheory.IsFiniteMeasure μ] (K : ) (_hK : 0 K) :
      ∃ (_lam : ), ∀ (_ρ₀ _ρ₁ : MeasureTheory.ProbabilityMeasure X) (t : ), 0 tt 1True

      Displacement convexity of entropy along Wasserstein geodesics

      Gradient flow structure for entropy functional

      Instances For

        Connection to PLFA framework: entropy provides F functional

        Equations
        Instances For

          Entropy functional satisfies convexity along geodesics (for PLFA)

          Entropy satisfies the Energy-Dissipation Equality (EDE)

          theorem Frourio.entropy_EVI {X : Type u_1} [MeasurableSpace X] [PseudoMetricSpace X] (μ : MeasureTheory.Measure X) [MeasureTheory.IsFiniteMeasure μ] (_K : ) :
          ∃ (_flow : EntropyGradientFlow X μ), ∀ (t : ), 0 t∀ (_ρ₀ : MeasureTheory.ProbabilityMeasure X), True

          Entropy satisfies Evolution Variational Inequality (EVI)

          JKO scheme for entropy: discrete gradient flow

          Equations
          Instances For

            JKO iterates converge to gradient flow as τ → 0

            Instance: Entropy functional for PLFA/EVI framework integration

            Equations
            Instances For