From 6d111b2d517e327ba9cf317556760c2c8e828310 Mon Sep 17 00:00:00 2001 From: herbelin Date: Wed, 27 Feb 2008 19:36:07 +0000 Subject: Application patch #1807 sur hypothèse inutile de Rpower_O MIME-Version: 1.0 Content-Type: text/plain; charset=UTF-8 Content-Transfer-Encoding: 8bit git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10599 85f007b7-540e-0410-9357-904b9bb8a0f7 --- CHANGES | 3 ++- theories/Reals/Rpower.v | 4 ++-- 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. -- cgit v1.2.3