Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
RemyDegenne committed Mar 25, 2024
1 parent b4c779a commit 681fa5e
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions TestingLowerBounds/Renyi.lean
Original file line number Diff line number Diff line change
Expand Up @@ -122,15 +122,15 @@ end FDiv
open Classical in
noncomputable def renyiDiv (a : ℝ) (μ ν : Measure α) : EReal :=
if a = 0 then - log (ν {x | 0 < (∂μ/∂ν) x}).toReal
else if a = 1 then klReal μ ν
else if a = 1 then EReal.toReal (kl μ ν)
else if fDiv (renyiFun a) μ ν ≠ ⊤
then (a - 1)⁻¹ * log (1 + (a - 1) * (fDiv (renyiFun a) μ ν).toReal)
else

lemma renyiDiv_zero (μ ν : Measure α) :
renyiDiv 0 μ ν = - log (ν {x | 0 < (∂μ/∂ν) x}).toReal := if_pos rfl

lemma renyiDiv_one (μ ν : Measure α) : renyiDiv 1 μ ν = klReal μ ν := by
lemma renyiDiv_one (μ ν : Measure α) : renyiDiv 1 μ ν = EReal.toReal (kl μ ν) := by
rw [renyiDiv, if_neg (by simp), if_pos rfl]

lemma renyiDiv_eq_top_iff_fDiv_eq_top [IsFiniteMeasure μ] [SigmaFinite ν]
Expand Down

0 comments on commit 681fa5e

Please sign in to comment.