aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-17 13:44:32 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-17 13:44:32 +0000
commitc710be6c4d2fda836939c404a1795e8a9171634e (patch)
treef3e88e762686b03d7d3a98655a7e2f75db652846 /theories/Bool
parente9ccfc401c610ce4df6b06f48c611070a26f89d7 (diff)
Kill some useless dependencies (Bvector, Program.Syntax)
Bvector uses only Minus, so let's avoid loading Arith (and hence ArithRing and hence parts of Z, N) Program.Syntax no longer need Lists now that list is in Datatypes. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12785 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool')
-rw-r--r--theories/Bool/Bvector.v5
1 files changed, 2 insertions, 3 deletions
diff --git a/theories/Bool/Bvector.v b/theories/Bool/Bvector.v
index 7ecfa43f2..d9da08672 100644
--- a/theories/Bool/Bvector.v
+++ b/theories/Bool/Bvector.v
@@ -10,9 +10,8 @@
(** Bit vectors. Contribution by Jean Duprat (ENS Lyon). *)
-Require Export Bool.
-Require Export Sumbool.
-Require Import Arith.
+Require Export Bool Sumbool.
+Require Import Minus.
Open Local Scope nat_scope.