aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-10-21 06:48:00 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-10-21 06:48:00 +0000
commitf0168fd8ce775b0a96e8cf026e953e9d55f4de25 (patch)
treeedbca2c262da236a72bfe5db54b7f700eb17d430 /theories/Arith
parent843bbc240d6ece54efc4f6f13035ef0ffac8f886 (diff)
Solve name conflict about pow introduced by commit 13546.
- NPeano isn't Exported by default anymore (contains pow for nat). - in coq_micromega.ml, we specify more where to find the pow of R. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13569 85f007b7-540e-0410-9357-904b9bb8a0f7
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.