aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/NArith/NArith.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-09 17:44:39 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-09 17:44:39 +0000
commit3453438833ff72ad991e0691207481cb6682f246 (patch)
tree0086295f174b75895779e7294c2963d33293d1f0 /theories/NArith/NArith.v
parent959b8555351fcf30bd747b47167dd0dca96d34c6 (diff)
NBinary improved, contains more, subsumes NOrderedType
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12715 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/NArith/NArith.v')
-rw-r--r--theories/NArith/NArith.v18
1 files changed, 17 insertions, 1 deletions
diff --git a/theories/NArith/NArith.v b/theories/NArith/NArith.v
index 53ba50ffe..3a87880ac 100644
--- a/theories/NArith/NArith.v
+++ b/theories/NArith/NArith.v
@@ -14,5 +14,21 @@ Require Export BinPos.
Require Export BinNat.
Require Export Nnat.
Require Export Ndigits.
-
Require Export NArithRing.
+Require NBinary Nminmax.
+
+Module N := NBinary.N <+ Nminmax.Nextend.
+
+(** [N] contains An [order] tactic for natural numbers *)
+
+(** Note that [N.order] is domain-agnostic: it will not prove
+ [1<=2] or [x<=x+x], but rather things like [x<=y -> y<=x -> x=y]. *)
+
+Local Open Scope N_scope.
+
+Section TestOrder.
+ Let test : forall x y, x<=y -> y<=x -> x=y.
+ Proof.
+ N.order.
+ Qed.
+End TestOrder.