aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zcomplements.v
diff options
context:
space:
mode:
authorGravatar bertot <bertot@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-10-05 13:27:01 +0000
committerGravatar bertot <bertot@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-10-05 13:27:01 +0000
commit3004d1c1d53a13c4ea34e1997367ad6e0b1c31eb (patch)
tree2abfa1b7a645d037f04d27189d295305c9a672dc /theories/ZArith/Zcomplements.v
parente85d10cc40e968ea3d16ca32a58ac4b3caf2b100 (diff)
revert, the previous commit was a mistake
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9214 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Zcomplements.v')
-rw-r--r--theories/ZArith/Zcomplements.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/Zcomplements.v b/theories/ZArith/Zcomplements.v
index e5c18bd33..a3f17f4d8 100644
--- a/theories/ZArith/Zcomplements.v
+++ b/theories/ZArith/Zcomplements.v
@@ -8,7 +8,7 @@
(*i $Id$ i*)
-Require Export ZArithRing.
+Require Import ZArithRing.
Require Import ZArith_base.
Require Import Omega.
Require Import Wf_nat.