aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sorting/Heap.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-03-14 20:27:40 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-03-14 20:27:40 +0000
commit125f04f251e62674379dfe9ae7ee660586e5c954 (patch)
tree357c16ee91c1567fafd5ad524b3ab87f684d6072 /theories/Sorting/Heap.v
parent9c699950feff3631c206f87f1d7d8c1686f1f597 (diff)
Suppress some warnings by writing ugly Coq.Relations.Relations in some .v
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10672 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Sorting/Heap.v')
-rw-r--r--theories/Sorting/Heap.v7
1 files changed, 1 insertions, 6 deletions
diff --git a/theories/Sorting/Heap.v b/theories/Sorting/Heap.v
index 573d5adb8..b75aee610 100644
--- a/theories/Sorting/Heap.v
+++ b/theories/Sorting/Heap.v
@@ -12,12 +12,7 @@
(* G. Huet 1-9-95 uses Multiset *)
-Require Import List.
-Require Import Multiset.
-Require Import Permutation.
-Require Import Relations.
-Require Import Sorting.
-
+Require Import List Multiset Permutation Coq.Relations.Relations Sorting.
Section defs.