aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-02-06 01:05:30 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-02-08 20:10:54 +0100
commitbd41c9d104550ad5472a28655cd6353ba6df1696 (patch)
tree3dbe7fb15b4b32d7350fe87aca29f7e977dad5ab
parent009fb68f0578e462b817f50772e2fba8d58c4f0d (diff)
Less dependencies in Omega.
-rw-r--r--plugins/omega/Omega.v2
-rw-r--r--plugins/setoid_ring/InitialRing.v3
-rw-r--r--theories/NArith/Nnat.v2
3 files changed, 3 insertions, 4 deletions
diff --git a/plugins/omega/Omega.v b/plugins/omega/Omega.v
index ea5a8cb71..7e7b52bb9 100644
--- a/plugins/omega/Omega.v
+++ b/plugins/omega/Omega.v
@@ -54,4 +54,4 @@ Hint Extern 10 (~ (_ < _)%Z) => abstract omega: zarith.
Hint Extern 10 (~ (_ >= _)%Z) => abstract omega: zarith.
Hint Extern 10 (~ (_ > _)%Z) => abstract omega: zarith.
-Hint Extern 10 False => abstract omega: zarith. \ No newline at end of file
+Hint Extern 10 False => abstract omega: zarith.
diff --git a/plugins/setoid_ring/InitialRing.v b/plugins/setoid_ring/InitialRing.v
index e805151ce..ca178dd38 100644
--- a/plugins/setoid_ring/InitialRing.v
+++ b/plugins/setoid_ring/InitialRing.v
@@ -6,8 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-Require Import ZArith_base.
-Require Import Zpow_def.
+Require Import Zbool.
Require Import BinInt.
Require Import BinNat.
Require Import Setoid.
diff --git a/theories/NArith/Nnat.v b/theories/NArith/Nnat.v
index 346169e7f..cddc5f4cf 100644
--- a/theories/NArith/Nnat.v
+++ b/theories/NArith/Nnat.v
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-Require Import Arith_base Compare_dec Sumbool Div2 Min Max.
+Require Import Minus Compare_dec Sumbool Div2 Min Max.
Require Import BinPos BinNat Pnat.
(** * Conversions from [N] to [nat] *)