aboutsummaryrefslogtreecommitdiffstats
path: root/lib/Maps.v
diff options
context:
space:
mode:
authorxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2011-08-19 09:13:09 +0000
committerxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2011-08-19 09:13:09 +0000
commit7ea8a55692e2a2d32efa0c84e19c37a3b56a0fd1 (patch)
treee324aff1a958e0a5d83f805ff3ca1d9eb07939f4 /lib/Maps.v
parent5b73a4f223a0cadb7df3f1320fed86cde0d67d6e (diff)
downloadcompcert-kvx-7ea8a55692e2a2d32efa0c84e19c37a3b56a0fd1.tar.gz
compcert-kvx-7ea8a55692e2a2d32efa0c84e19c37a3b56a0fd1.zip
Cleaned up old commented-out parts
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1719 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'lib/Maps.v')
-rw-r--r--lib/Maps.v5
1 files changed, 0 insertions, 5 deletions
diff --git a/lib/Maps.v b/lib/Maps.v
index 793c2231..f8d1bd5a 100644
--- a/lib/Maps.v
+++ b/lib/Maps.v
@@ -998,11 +998,6 @@ Module PTree <: TREE.
destruct H0. congruence.
Qed.
-(*
- Definition fold (A B : Type) (f: B -> positive -> A -> B) (tr: t A) (v: B) :=
- List.fold_left (fun a p => f a (fst p) (snd p)) (elements tr) v.
-*)
-
Fixpoint xfold (A B: Type) (f: B -> positive -> A -> B)
(i: positive) (m: t A) (v: B) {struct m} : B :=
match m with