aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-29 22:11:18 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-29 22:11:18 +0000
commitd93a43901ff6a4bd264383df486f2dd1387157e6 (patch)
treeb07154b325664720cc334716c820a203720ceec2 /theories
parent37b2a9827f241357169615b8a489958c118b579b (diff)
niveau 49 devient next
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4091 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r--theories/Reals/Rsyntax.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/theories/Reals/Rsyntax.v b/theories/Reals/Rsyntax.v
index a008cd06e..60a205cfd 100644
--- a/theories/Reals/Rsyntax.v
+++ b/theories/Reals/Rsyntax.v
@@ -222,19 +222,19 @@ Notation "- x" := (Ropp x) (at level 0) : R_scope
V8only (at level 40, left associativity).
Notation "x == y == z" := (eqT R x y)/\(eqT R y z)
(at level 5, y at level 4, no associtivity): R_scope
- V8only (at level 50, y at level 49, no associativity).
+ V8only (at level 50, y at next level, no associativity).
Notation "x <= y <= z" := (Rle x y)/\(Rle y z)
(at level 5, y at level 4) : R_scope
- V8only (at level 50, y at level 49, no associativity).
+ V8only (at level 50, y at next level, no associativity).
Notation "x <= y < z" := (Rle x y)/\(Rlt y z)
(at level 5, y at level 4) : R_scope
- V8only (at level 50, y at level 49, no associativity).
+ V8only (at level 50, y at next level, no associativity).
Notation "x < y < z" := (Rlt x y)/\(Rlt y z)
(at level 5, y at level 4) : R_scope
- V8only (at level 50, y at level 49, no associativity).
+ V8only (at level 50, y at next level, no associativity).
Notation "x < y <= z" := (Rlt x y)/\(Rle y z)
(at level 5, y at level 4) : R_scope
- V8only (at level 50, y at level 49, no associativity).
+ V8only (at level 50, y at next level, no associativity).
(*Notation "x <> y" := ~(eqT R x y) (at level 5) : R_scope.*)
Notation "/ x" := (Rinv x) (at level 0): R_scope
V8only (at level 30, left associativity).