aboutsummaryrefslogtreecommitdiff
path: root/src/Util/ListUtil
diff options
context:
space:
mode:
authorGravatar Jason Gross <jagro@google.com>2018-08-13 19:20:04 -0400
committerGravatar Jason Gross <jagro@google.com>2018-08-13 19:20:04 -0400
commit766e4bd7ae4f299dcd159216813062a93c58c2c3 (patch)
tree22945e49c269f526e25b23bccdc2a340c8f16784 /src/Util/ListUtil
parentdcdd233f666fbeab71bb25a6f48bcf3b7d36cbcd (diff)
Move a lemma
Diffstat (limited to 'src/Util/ListUtil')
-rw-r--r--src/Util/ListUtil/FoldBool.v12
1 files changed, 12 insertions, 0 deletions
diff --git a/src/Util/ListUtil/FoldBool.v b/src/Util/ListUtil/FoldBool.v
index b69081cab..f6cac6118 100644
--- a/src/Util/ListUtil/FoldBool.v
+++ b/src/Util/ListUtil/FoldBool.v
@@ -55,3 +55,15 @@ Proof.
intuition (congruence || (subst; auto)).
apply (H1 (_, _)); auto.
Qed.
+
+Lemma fold_andb_map_snoc A B f x xs y ys
+ : @fold_andb_map A B f (xs ++ [x]) (ys ++ [y]) = @fold_andb_map A B f xs ys && f x y.
+Proof.
+ clear.
+ revert ys; induction xs as [|x' xs'], ys as [|y' ys']; cbn;
+ rewrite ?Bool.andb_true_r, ?Bool.andb_false_r;
+ try (destruct ys'; cbn; rewrite Bool.andb_false_r);
+ try (destruct xs'; cbn; rewrite Bool.andb_false_r);
+ try reflexivity.
+ rewrite IHxs', Bool.andb_assoc; reflexivity.
+Qed.