From e7a09d51d6f96f59e427a079fcbe7942edd330f1 Mon Sep 17 00:00:00 2001 From: herbelin Date: Sun, 21 Sep 2003 22:43:12 +0000 Subject: Les notations 'x <= y <= z' sont réservées et s'appliquent maintenant aussi à nat MIME-Version: 1.0 Content-Type: text/plain; charset=UTF-8 Content-Transfer-Encoding: 8bit git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4428 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Init/Peano.v | 7 +++++++ 1 file changed, 7 insertions(+) (limited to 'theories') 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). -- cgit v1.2.3