aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rpower.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-29 18:55:04 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-29 18:55:04 +0000
commit855cc609d2888ef59d848ed688f02390811b28c7 (patch)
treebaf4ca25b36b88f2e77a979b6ac61c04b49255e1 /theories/Reals/Rpower.v
parentd4e5e38cffdd29a9af0e8762fc1f49a817944743 (diff)
Argumentation plus poussée de pourquoi on retire la condition x>0 dans
Rpower_O alors qu'on la garde pour les autres propriétés de la puissance. (résultat d'une discussion avec Assia et Jean-Marc) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10609 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Rpower.v')
-rw-r--r--theories/Reals/Rpower.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/theories/Reals/Rpower.v b/theories/Reals/Rpower.v
index 61cd98e56..701ed449b 100644
--- a/theories/Reals/Rpower.v
+++ b/theories/Reals/Rpower.v
@@ -403,6 +403,9 @@ Infix Local "^R" := Rpower (at level 30, right associativity) : R_scope.
(** * Properties of Rpower *)
(******************************************************************)
+(** Note: Because [ln] is artificially prolongated to 1 on negative
+ reals, no side condition is needed to state "x ^R 0 = 1" *)
+
Theorem Rpower_plus : forall x y z:R, z ^R (x + y) = z ^R x * z ^R y.
Proof.
intros x y z; unfold Rpower in |- *.