Skip to content

Commit

Permalink
Lemma gt0_ltr_powR
Browse files Browse the repository at this point in the history
  • Loading branch information
hoheinzollern committed Sep 23, 2023
1 parent de6bdd5 commit 380181e
Show file tree
Hide file tree
Showing 2 changed files with 13 additions and 0 deletions.
3 changes: 3 additions & 0 deletions CHANGELOG_UNRELEASED.md
Original file line number Diff line number Diff line change
Expand Up @@ -70,6 +70,9 @@
- in `measure.v`:
+ definition `ess_sup`, lemma `ess_sup_ge0`

- in `exp.v`:
+ lemma `gt0_ltr_powR`

### Changed

- `mnormalize` moved from `kernel.v` to `measure.v` and generalized
Expand Down
10 changes: 10 additions & 0 deletions theories/exp.v
Original file line number Diff line number Diff line change
Expand Up @@ -676,6 +676,16 @@ move=> /predU1P[->//|xy]; first by rewrite eqxx.
by apply/orP; right; rewrite /powR !gt_eqF// ltr_expR ltr_pmul2l// ltr_ln.
Qed.

Lemma gt0_ltr_powR (r : R) : 0 < r ->
{in `[0, +oo[ &, {homo powR ^~ r : x y / x < y >-> x < y}}.
Proof.
move=> r0 x y; rewrite !in_itv/= !andbT !le_eqVlt => /predU1P[<-|x0].
move=> /predU1P[<-|y0 _]; first by rewrite ltxx//.
by rewrite powR0 ?(gt_eqF r0)// powR_gt0.
move=> /predU1P[<-|y0]; first rewrite ltNge ltW//.
by rewrite /powR !gt_eqF// ltr_expR ltr_pmul2l// ltr_ln.
Qed.

Lemma powRM x y r : 0 <= x -> 0 <= y -> (x * y) `^ r = x `^ r * y `^ r.
Proof.
rewrite /powR mulf_eq0.
Expand Down

0 comments on commit 380181e

Please sign in to comment.