aboutsummaryrefslogtreecommitdiff
path: root/src/Util/Tuple.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-04-28 13:11:33 -0400
committerGravatar Jason Gross <jgross@mit.edu>2017-04-28 13:11:33 -0400
commit05c101daeef6358bfc64e5997c8b8aea7d03f30d (patch)
tree09ed06bd363c4f7817c2e12560372965a6ff0af0 /src/Util/Tuple.v
parent920dbb90413ecf64424799e2eec15dbc02d1dbfb (diff)
Fix nth_default for the tip of v8.6
This is bug #5497, https://coq.inria.fr/bugs/show_bug.cgi?id=5497, Coq v8.6 has weaker pattern matching than Coq 8.6 (regression)
Diffstat (limited to 'src/Util/Tuple.v')
-rw-r--r--src/Util/Tuple.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/src/Util/Tuple.v b/src/Util/Tuple.v
index 763765898..cf3ce377e 100644
--- a/src/Util/Tuple.v
+++ b/src/Util/Tuple.v
@@ -780,11 +780,11 @@ Lemma map_append {A B n} (f:A->B) : forall (x:tuple A n) (a:A),
map f (append a x) = append (f a) (map f x).
Proof. destruct n; auto using map_append'. Qed.
-Fixpoint nth_default {A m} (d:A) n (x: tuple A m) : A :=
- match m,n with
- | O, _ => d
- | S m', O => hd x
- | S m', S n' => nth_default d n' (tl x)
+Fixpoint nth_default {A m} (d:A) n : tuple A m -> A :=
+ match m, n with
+ | O, _ => fun _ => d
+ | S m', O => hd
+ | S m', S n' => fun x => nth_default d n' (tl x)
end.
(* map operation that carries state *)