aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-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).