aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories7
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-01-09 14:42:52 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-01-09 14:42:52 +0000
commiteb2f9b5023f6d42f89ddfb3927fda81d6cb334a1 (patch)
treeb78fc74d3f0258dce8bbbc6cc747f0a77ed6f208 /theories7
parent4bc8229e325cbddc26c7c73157d5e163fd00f2ad (diff)
Retrait de la notation '^' pour 'power' en V7 car sinon confusion avec la syntaxe '^' de append qui est a un autre niveau
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5188 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories7')
-rw-r--r--theories7/Reals/Rfunctions.v2
-rw-r--r--theories7/ZArith/Zpower.v4
2 files changed, 3 insertions, 3 deletions
diff --git a/theories7/Reals/Rfunctions.v b/theories7/Reals/Rfunctions.v
index b283b9fd8..1cc327537 100644
--- a/theories7/Reals/Rfunctions.v
+++ b/theories7/Reals/Rfunctions.v
@@ -70,7 +70,7 @@ Fixpoint pow [r:R;n:nat]:R:=
|(S n) => (Rmult r (pow r n))
end.
-Infix "^" pow (at level 2, left associativity) : R_scope V8only.
+V8Infix "^" pow : R_scope.
Lemma pow_O: (x : R) (pow x O) == R1.
Proof.
diff --git a/theories7/ZArith/Zpower.v b/theories7/ZArith/Zpower.v
index 73e8a08da..dbfdf2229 100644
--- a/theories7/ZArith/Zpower.v
+++ b/theories7/ZArith/Zpower.v
@@ -73,7 +73,7 @@ Definition Zpower :=
| (NEG p) => `0`
end.
-Infix "^" Zpower (at level 2, left associativity) : Z_scope V8only.
+V8Infix "^" Zpower : Z_scope.
Hints Immediate Zpower_nat_is_exp : zarith.
Hints Immediate Zpower_pos_is_exp : zarith.
@@ -93,7 +93,7 @@ End section1.
(* Exporting notation "^" *)
-Infix "^" Zpower (at level 2, left associativity) : Z_scope V8only.
+V8Infix "^" Zpower : Z_scope.
Hints Immediate Zpower_nat_is_exp : zarith.
Hints Immediate Zpower_pos_is_exp : zarith.