aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2017-04-29 09:09:35 +0200
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2017-04-29 09:09:35 +0200
commit991b78fd9627ee76f1a1a39b8460bf361c6af53d (patch)
treed60509f670af57ae8f50374632977ec019b67bfa /theories/Reals
parent1c8ed18d5f67d7d5656342584b8dcf8a441cb87f (diff)
Suppress warning message in stdlib.
Diffstat (limited to 'theories/Reals')
-rw-r--r--theories/Reals/Rfunctions.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Reals/Rfunctions.v b/theories/Reals/Rfunctions.v
index 653fac8d9..606136333 100644
--- a/theories/Reals/Rfunctions.v
+++ b/theories/Reals/Rfunctions.v
@@ -704,7 +704,7 @@ Lemma powerRZ_ind (P : Z -> R -> R -> Prop) :
forall x (m : Z), P m x (powerRZ x m)%R.
Proof.
intros ? ? ? x m.
- destruct (intP m) as [n Hm| n Hm|n Hm].
+ destruct (intP m) as [Hm|n Hm|n Hm].
- easy.
- now rewrite <- pow_powerRZ.
- unfold powerRZ.