aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--CHANGES3
-rw-r--r--theories/Reals/Rpower.v4
2 files changed, 4 insertions, 3 deletions
diff --git a/CHANGES b/CHANGES
index 817978b74..e93eb275c 100644
--- a/CHANGES
+++ b/CHANGES
@@ -53,7 +53,8 @@ Libraries
as "Immediate". A compatibility "oldset" database retains these expensive
hints, so using "(e)auto with set oldset" should help porting scripts.
Same for FSetWeakInterface and FMap(Weak)Interface.
-- Few changes in Reals (lemmas on prod_f_SO now on prod_f_R0).
+- Few changes in Reals (lemmas on prod_f_SO now on prod_f_R0, useless
+ assumption in Rpower_O removed).
- Slight restructuration of the Logic library regarding choice and classical
logic. Addition of files providing intuitionistic axiomatizations of
descriptions: Epsilon.v, Description.v and IndefiniteDescription.v
diff --git a/theories/Reals/Rpower.v b/theories/Reals/Rpower.v
index 5c1c07c73..61cd98e56 100644
--- a/theories/Reals/Rpower.v
+++ b/theories/Reals/Rpower.v
@@ -418,9 +418,9 @@ Proof.
ring.
Qed.
-Theorem Rpower_O : forall x:R, 0 < x -> x ^R 0 = 1.
+Theorem Rpower_O : forall x:R, x ^R 0 = 1.
Proof.
- intros x H; unfold Rpower in |- *.
+ intros x; unfold Rpower in |- *.
rewrite Rmult_0_l; apply exp_0.
Qed.