diff options
author | barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2006-10-27 21:21:17 +0000 |
---|---|---|
committer | barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2006-10-27 21:21:17 +0000 |
commit | 5b8e645b675b6b2efac8e13c29da5e984248e507 (patch) | |
tree | f39598f12eefa82801eb3adb9b954edf4b56cadc /theories/ZArith | |
parent | c5e8c731ede28ba4f734bbd143c7d7e5a05c365a (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')
-rw-r--r-- | theories/ZArith/Zabs.v | 4 | ||||
-rw-r--r-- | theories/ZArith/Zmax.v | 2 | ||||
-rw-r--r-- | theories/ZArith/Zmin.v | 2 | ||||
-rw-r--r-- | theories/ZArith/Znat.v | 2 | ||||
-rw-r--r-- | theories/ZArith/Zorder.v | 2 | ||||
-rw-r--r-- | theories/ZArith/auxiliary.v | 2 |
6 files changed, 7 insertions, 7 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. diff --git a/theories/ZArith/Zmax.v b/theories/ZArith/Zmax.v index ca647ff3c..b2c068564 100644 --- a/theories/ZArith/Zmax.v +++ b/theories/ZArith/Zmax.v @@ -7,7 +7,7 @@ (************************************************************************) (*i $Id$ i*) -Require Import Arith. +Require Import Arith_base. Require Import BinInt. Require Import Zcompare. Require Import Zorder. diff --git a/theories/ZArith/Zmin.v b/theories/ZArith/Zmin.v index a1e46fa5f..0e0caa1bd 100644 --- a/theories/ZArith/Zmin.v +++ b/theories/ZArith/Zmin.v @@ -12,7 +12,7 @@ from Russell O'Connor (Radbout U., Nijmegen, The Netherlands). *) -Require Import Arith. +Require Import Arith_base. Require Import BinInt. Require Import Zcompare. Require Import Zorder. diff --git a/theories/ZArith/Znat.v b/theories/ZArith/Znat.v index 8a18798c2..27f31bf83 100644 --- a/theories/ZArith/Znat.v +++ b/theories/ZArith/Znat.v @@ -10,7 +10,7 @@ (** Binary Integers (Pierre Crégut, CNET, Lannion, France) *) -Require Export Arith. +Require Export Arith_base. Require Import BinPos. Require Import BinInt. Require Import Zcompare. diff --git a/theories/ZArith/Zorder.v b/theories/ZArith/Zorder.v index e26754505..4b0d2562e 100644 --- a/theories/ZArith/Zorder.v +++ b/theories/ZArith/Zorder.v @@ -11,7 +11,7 @@ Require Import BinPos. Require Import BinInt. -Require Import Arith. +Require Import Arith_base. Require Import Decidable. Require Import Zcompare. diff --git a/theories/ZArith/auxiliary.v b/theories/ZArith/auxiliary.v index c6b398110..18b49f4bb 100644 --- a/theories/ZArith/auxiliary.v +++ b/theories/ZArith/auxiliary.v @@ -10,7 +10,7 @@ (** Binary Integers (Pierre Crégut, CNET, Lannion, France) *) -Require Export Arith. +Require Export Arith_base. Require Import BinInt. Require Import Zorder. Require Import Decidable. |