Zulip Chat Archive
Stream: Is there code for X?
Topic: ENNReal.rpow_ofNNReal
Michael Rothgang (Feb 11 2025 at 15:26):
I have one sorry in branch#MR-generalise-enorm-6 which would be closed by the following statement. Is this really missing from mathlib?
theorem ENNReal.rpow_ofNNReal {M : ℝ≥0} {P : ℝ} :
(ENNReal.ofNNReal M).rpow P = ENNReal.ofNNReal (M ^ P) := sorry
Ruben Van de Velde (Feb 11 2025 at 15:37):
import Mathlib
open NNReal
theorem ENNReal.rpow_ofNNReal {M : ℝ≥0} {P : ℝ} :
(ENNReal.ofNNReal M) ^ P = ENNReal.ofNNReal (M ^ P) := by
rw [coe_rpow_def]
-- ⊢ (if M = 0 ∧ P < 0 then ⊤ else ↑(M ^ P)) = ↑(M ^ P)
Seems like it's false
Andrew Yang (Feb 11 2025 at 15:40):
docs#ENNReal.coe_rpow_of_nonneg
Yaël Dillies (Feb 11 2025 at 15:52):
.. which btw is the wrong way around
Michael Rothgang (Feb 11 2025 at 20:30):
If you submit a PR renaming it, I'll happily review it.
Last updated: May 02 2025 at 03:31 UTC