aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/RIneq.v
diff options
context:
space:
mode:
authorGravatar Yves Bertot <Yves.Bertot@inria.fr>2017-09-06 08:39:06 +0200
committerGravatar Yves Bertot <Yves.Bertot@inria.fr>2017-09-06 08:39:06 +0200
commit2d137819572c4307b34bfdbdcf4ad0dc9ab240f3 (patch)
tree143870f1d7962715d23927e4d09c25d9a2327f79 /theories/Reals/RIneq.v
parentdf6ae3d59af8f880a0411217b8e6f0dae0b92133 (diff)
changed statements of Rpower_lt and Rle_power and added
Rlt_Rpower_l and pow_INR. Unfortunately theorems Rpower_lt and Rle_power are named inconsistently, in spite of their similarity.
Diffstat (limited to 'theories/Reals/RIneq.v')
-rw-r--r--theories/Reals/RIneq.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/theories/Reals/RIneq.v b/theories/Reals/RIneq.v
index 7bcd2799a..bc82c3712 100644
--- a/theories/Reals/RIneq.v
+++ b/theories/Reals/RIneq.v
@@ -1611,6 +1611,9 @@ Proof.
Qed.
Hint Resolve mult_INR: real.
+Lemma pow_INR (m n: nat) : INR (m ^ n) = pow (INR m) n.
+Proof. now induction n as [|n IHn];[ | simpl; rewrite mult_INR, IHn]. Qed.
+
(*********)
Lemma lt_0_INR : forall n:nat, (0 < n)%nat -> 0 < INR n.
Proof.