Skip to content

Commit

Permalink
feat(analysis/special_functions/pow): add ennreal.to_nnreal_rpow (#5042)
Browse files Browse the repository at this point in the history
cut ennreal.to_real_rpow into two lemmas: to_nnreal_rpow and to_real_rpow
  • Loading branch information
RemyDegenne committed Nov 20, 2020
1 parent de76acd commit 8d40e8d
Showing 1 changed file with 4 additions and 2 deletions.
6 changes: 4 additions & 2 deletions src/analysis/special_functions/pow.lean
Expand Up @@ -1422,8 +1422,7 @@ begin
nnreal.one_le_rpow_of_pos_of_le_one_of_nonpos hx1 hx2 (le_of_lt hz)],
end

lemma to_real_rpow (x : ennreal) (z : ℝ) :
(x.to_real) ^ z = (x ^ z).to_real :=
lemma to_nnreal_rpow (x : ennreal) (z : ℝ) : (x.to_nnreal) ^ z = (x ^ z).to_nnreal :=
begin
rcases lt_trichotomy z 0 with H|H|H,
{ cases x, { simp [H, ne_of_lt] },
Expand All @@ -1435,6 +1434,9 @@ begin
simp [coe_rpow_of_nonneg _ (le_of_lt H)] }
end

lemma to_real_rpow (x : ennreal) (z : ℝ) : (x.to_real) ^ z = (x ^ z).to_real :=
by rw [ennreal.to_real, ennreal.to_real, ←nnreal.coe_rpow, ennreal.to_nnreal_rpow]

end ennreal

section measurability_ennreal
Expand Down

0 comments on commit 8d40e8d

Please sign in to comment.