From c710be6c4d2fda836939c404a1795e8a9171634e Mon Sep 17 00:00:00 2001 From: letouzey Date: Wed, 17 Feb 2010 13:44:32 +0000 Subject: 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 --- theories/Bool/Bvector.v | 5 ++--- 1 file changed, 2 insertions(+), 3 deletions(-) (limited to 'theories/Bool') 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. -- cgit v1.2.3