aboutsummaryrefslogtreecommitdiffstats
path: root/lib/Maps.v
diff options
context:
space:
mode:
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