aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Structures
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-09 17:44:52 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-09 17:44:52 +0000
commitbf90d39cec401f5daad2eb26c915ceba65e1a5cc (patch)
treeee1eb266a33d1f9d16af1268136f60ee72c5bc04 /theories/Structures
parent38dac30c6877122634e7b34ec7cd1b6ab2b67ebb (diff)
NPeano improved, subsumes NatOrderedType
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12717 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Structures')
-rw-r--r--theories/Structures/OrdersEx.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Structures/OrdersEx.v b/theories/Structures/OrdersEx.v
index 90840ce1f..b0702f681 100644
--- a/theories/Structures/OrdersEx.v
+++ b/theories/Structures/OrdersEx.v
@@ -13,7 +13,7 @@
(* $Id$ *)
-Require Import Orders NatOrderedType POrderedType NArith
+Require Import Orders NPeano POrderedType NArith
ZArith RelationPairs EqualitiesFacts.
(** * Examples of Ordered Type structures. *)
@@ -21,7 +21,7 @@ Require Import Orders NatOrderedType POrderedType NArith
(** Ordered Type for [nat], [Positive], [N], [Z] with the usual order. *)
-Module Nat_as_OT := NatOrderedType.Nat_as_OT.
+Module Nat_as_OT := NPeano.Nat.
Module Positive_as_OT := POrderedType.Positive_as_OT.
Module N_as_OT := NArith.N.
Module Z_as_OT := ZArith.Z.