aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-10-05 10:12:15 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-10-05 10:12:15 +0000
commit4524219d80c2d5ea50ca8bba819bbc14bd6b9988 (patch)
treef5204b39bba079321a8c6a21d400f5f84f9d9c91 /theories/Arith
parent685d10fa1691ced3b44f77ae8587e0b27f57810b (diff)
Arith NArith et ZArith exportent ring + nettoyage dans Ring_polynom
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9210 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith')
-rw-r--r--theories/Arith/Arith.v2
-rw-r--r--theories/Arith/Min.v2
2 files changed, 3 insertions, 1 deletions
diff --git a/theories/Arith/Arith.v b/theories/Arith/Arith.v
index b076de2af..c522e01b3 100644
--- a/theories/Arith/Arith.v
+++ b/theories/Arith/Arith.v
@@ -18,3 +18,5 @@ Require Export Between.
Require Export Peano_dec.
Require Export Compare_dec.
Require Export Factorial.
+
+Require Export ArithRing.
diff --git a/theories/Arith/Min.v b/theories/Arith/Min.v
index 3e64980cb..d86d7f116 100644
--- a/theories/Arith/Min.v
+++ b/theories/Arith/Min.v
@@ -8,7 +8,7 @@
(*i $Id$ i*)
-Require Import Arith.
+Require Import Le.
Open Local Scope nat_scope.