aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zabs.v
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-10-27 21:21:17 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-10-27 21:21:17 +0000
commit5b8e645b675b6b2efac8e13c29da5e984248e507 (patch)
treef39598f12eefa82801eb3adb9b954edf4b56cadc /theories/ZArith/Zabs.v
parentc5e8c731ede28ba4f734bbd143c7d7e5a05c365a (diff)
simplif de la partie ML de ring/field
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9302 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Zabs.v')
-rw-r--r--theories/ZArith/Zabs.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/ZArith/Zabs.v b/theories/ZArith/Zabs.v
index f648867aa..c7f0bb723 100644
--- a/theories/ZArith/Zabs.v
+++ b/theories/ZArith/Zabs.v
@@ -9,7 +9,7 @@
(** Binary Integers (Pierre Crégut (CNET, Lannion, France) *)
-Require Import Arith.
+Require Import Arith_base.
Require Import BinPos.
Require Import BinInt.
Require Import Zorder.
@@ -127,4 +127,4 @@ Proof.
compute in |- *. intro H0. discriminate H0. intuition.
intros. absurd (0 <= Zneg p). compute in |- *. auto with arith. intuition.
-Qed. \ No newline at end of file
+Qed.