aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Arith')
-rw-r--r--theories/Arith/Max.v2
-rw-r--r--theories/Arith/Min.v2
2 files changed, 2 insertions, 2 deletions
diff --git a/theories/Arith/Max.v b/theories/Arith/Max.v
index 2022331bb..77dfa5080 100644
--- a/theories/Arith/Max.v
+++ b/theories/Arith/Max.v
@@ -8,7 +8,7 @@
(** THIS FILE IS DEPRECATED. Use [NPeano.Nat] instead. *)
-Require Export NPeano.
+Require Import NPeano.
Local Open Scope nat_scope.
Implicit Types m n p : nat.
diff --git a/theories/Arith/Min.v b/theories/Arith/Min.v
index 742c8126c..2b2cf860d 100644
--- a/theories/Arith/Min.v
+++ b/theories/Arith/Min.v
@@ -8,7 +8,7 @@
(** THIS FILE IS DEPRECATED. Use [NPeano.Nat] instead. *)
-Require Export NPeano.
+Require Import NPeano.
Open Local Scope nat_scope.
Implicit Types m n p : nat.