aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-07 08:44:10 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-07 08:44:10 +0000
commit027fb68b3c9014f66a7e75255b5769f414d14655 (patch)
tree4ed13c770b6dd34a50ebd461740878337fcb5f24 /theories/Reals
parentfdfe1e7d6cf663e1cc901d67b7cb1a477eab196d (diff)
Espaces superflus
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3853 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals')
-rw-r--r--theories/Reals/Rsyntax.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/theories/Reals/Rsyntax.v b/theories/Reals/Rsyntax.v
index 60befa9da..8b209bde2 100644
--- a/theories/Reals/Rsyntax.v
+++ b/theories/Reals/Rsyntax.v
@@ -221,16 +221,16 @@ Notation "- x" := (Ropp x) (at level 0) : R_scope
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).
-Notation "x <= y <= z" := (Rle x y)/\(Rle y z)
+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).
-Notation "x <= y < z" := (Rle x y)/\(Rlt y z)
+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).
-Notation "x < y < z" := (Rlt x y)/\(Rlt y z)
+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).
-Notation "x < y <= z" := (Rlt x y)/\(Rle y z)
+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).
Notation "x <> y" := ~(eqT R x y) (at level 5) : R_scope.