aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-09-26 12:13:06 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-09-26 12:13:06 +0000
commit4aec8fda1161953cf929b4e282eea9b672ab4058 (patch)
treeeea4b8ab24fdea8fb05206b1764ce1ed3c752d72 /theories/ZArith
parent351a500eada776832ac9b09657e42f5d6cd7210f (diff)
commit de field + renommages
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9179 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith')
-rw-r--r--theories/ZArith/Zcomplements.v3
-rw-r--r--theories/ZArith/Zdiv.v2
-rw-r--r--theories/ZArith/Znumtheory.v2
-rw-r--r--theories/ZArith/Zsqrt.v2
4 files changed, 4 insertions, 5 deletions
diff --git a/theories/ZArith/Zcomplements.v b/theories/ZArith/Zcomplements.v
index 718ac3b03..a3f17f4d8 100644
--- a/theories/ZArith/Zcomplements.v
+++ b/theories/ZArith/Zcomplements.v
@@ -8,8 +8,7 @@
(*i $Id$ i*)
-Require Import NewZArithRing.
-
+Require Import ZArithRing.
Require Import ZArith_base.
Require Import Omega.
Require Import Wf_nat.
diff --git a/theories/ZArith/Zdiv.v b/theories/ZArith/Zdiv.v
index 52f85eada..d08515e62 100644
--- a/theories/ZArith/Zdiv.v
+++ b/theories/ZArith/Zdiv.v
@@ -22,7 +22,7 @@ Then only after proves the main required property.
Require Export ZArith_base.
Require Import Zbool.
Require Import Omega.
-Require Import NewZArithRing.
+Require Import ZArithRing.
Require Import Zcomplements.
Open Local Scope Z_scope.
diff --git a/theories/ZArith/Znumtheory.v b/theories/ZArith/Znumtheory.v
index 14bfa6357..9ae354eae 100644
--- a/theories/ZArith/Znumtheory.v
+++ b/theories/ZArith/Znumtheory.v
@@ -9,7 +9,7 @@
(*i $Id$ i*)
Require Import ZArith_base.
-Require Import NewZArithRing.
+Require Import ZArithRing.
Require Import Zcomplements.
Require Import Zdiv.
Require Import Ndigits.
diff --git a/theories/ZArith/Zsqrt.v b/theories/ZArith/Zsqrt.v
index 3d57561ea..804ab679d 100644
--- a/theories/ZArith/Zsqrt.v
+++ b/theories/ZArith/Zsqrt.v
@@ -8,7 +8,7 @@
(* $Id$ *)
-Require Import NewZArithRing.
+Require Import ZArithRing.
Require Import Omega.
Require Export ZArith_base.
Open Local Scope Z_scope.