aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Structures
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Structures')
-rw-r--r--theories/Structures/OrdersEx.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Structures/OrdersEx.v b/theories/Structures/OrdersEx.v
index ffc5b91bc..2cb591968 100644
--- a/theories/Structures/OrdersEx.v
+++ b/theories/Structures/OrdersEx.v
@@ -21,7 +21,7 @@ Require Import Orders NPeano POrderedType NArith
Module Nat_as_OT := NPeano.Nat.
Module Positive_as_OT := POrderedType.Positive_as_OT.
-Module N_as_OT := NArith.N.
+Module N_as_OT := BinNat.N.
Module Z_as_OT := ZBinary.Z.
(** An OrderedType can now directly be seen as a DecidableType *)