aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-21 22:43:12 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-21 22:43:12 +0000
commite7a09d51d6f96f59e427a079fcbe7942edd330f1 (patch)
tree7417d4583ff73d0956aba0013b4eb4fb592dfc30 /theories
parent45a33238f36b0d3ced493f83c2db9b9e150a214f (diff)
Les notations 'x <= y <= z' sont réservées et s'appliquent maintenant aussi à nat
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4428 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rwxr-xr-xtheories/Init/Peano.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/theories/Init/Peano.v b/theories/Init/Peano.v
index eaa9256e5..e5b516090 100755
--- a/theories/Init/Peano.v
+++ b/theories/Init/Peano.v
@@ -28,6 +28,8 @@ Require Logic.
Require LogicSyntax.
Require Datatypes.
+Open Local Scope nat_scope.
+
Definition eq_S := (f_equal nat nat S).
Hint eq_S : v62 := Resolve (f_equal nat nat S).
@@ -172,6 +174,11 @@ Hints Unfold gt : core v62.
V8Infix ">" gt : nat_scope.
+V8Notation "x <= y <= z" := (le x y)/\(le y z) : nat_scope.
+V8Notation "x <= y < z" := (le x y)/\(lt y z) : nat_scope.
+V8Notation "x < y < z" := (lt x y)/\(lt y z) : nat_scope.
+V8Notation "x < y <= z" := (lt x y)/\(le y z) : nat_scope.
+
(** Pattern-Matching on natural numbers *)
Theorem nat_case : (n:nat)(P:nat->Prop)(P O)->((m:nat)(P (S m)))->(P n).