aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rfunctions.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-10 19:31:54 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-10 19:31:54 +0000
commitec6e25000ec0be1aaf3945eabaf5db670f0d1ece (patch)
tree91830ce02469fa8d80062bf726ea33541c786012 /theories/Reals/Rfunctions.v
parente71f85b0e48d5dc56c0da8277e78fa2c2d14aa50 (diff)
Notation '^'
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4586 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Rfunctions.v')
-rw-r--r--theories/Reals/Rfunctions.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/theories/Reals/Rfunctions.v b/theories/Reals/Rfunctions.v
index 3ea74f862..e9316e1ad 100644
--- a/theories/Reals/Rfunctions.v
+++ b/theories/Reals/Rfunctions.v
@@ -67,6 +67,8 @@ Fixpoint pow [r:R;n:nat]:R:=
|(S n) => (Rmult r (pow r n))
end.
+Infix "^" pow (at level 2, left associativity) : R_scope.
+
Lemma pow_O: (e : R) (pow e O) == R1.
Simpl; Auto with real.
Qed.