aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rtrigo_def.v
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/Reals/Rtrigo_def.v
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/Reals/Rtrigo_def.v')
-rw-r--r--theories/Reals/Rtrigo_def.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Reals/Rtrigo_def.v b/theories/Reals/Rtrigo_def.v
index 27393c265..c64931353 100644
--- a/theories/Reals/Rtrigo_def.v
+++ b/theories/Reals/Rtrigo_def.v
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-Require Import Max Rbase Rfunctions SeqSeries Rtrigo_fun.
+Require Import Rbase Rfunctions SeqSeries Rtrigo_fun Max.
Open Local Scope R_scope.
(********************************)