aboutsummaryrefslogtreecommitdiff
path: root/src/Util/Tuple.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-11-10 14:51:57 -0500
committerGravatar Jason Gross <jgross@mit.edu>2016-11-10 14:52:25 -0500
commitc19c7aa0b4efa8a2529304d4c4e46435d765699e (patch)
tree828b4fd8b4203170973106c8be660682672fbbfd /src/Util/Tuple.v
parent497ac4e2e7e331c48eddfd428f2287c5384c9c08 (diff)
Add Tuple and HList lemmas
Diffstat (limited to 'src/Util/Tuple.v')
-rw-r--r--src/Util/Tuple.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/src/Util/Tuple.v b/src/Util/Tuple.v
index 79747ec2d..d1dcbca30 100644
--- a/src/Util/Tuple.v
+++ b/src/Util/Tuple.v
@@ -195,6 +195,10 @@ Proof.
simpl @List.map.
Admitted.
+Lemma map_to_list {A B n ts} (f : A -> B)
+ : List.map f (@to_list A n ts) = @to_list B n (map f ts).
+Proof. Admitted.
+
Definition on_tuple2 {A B C} (f : list A -> list B -> list C) {a b c : nat}
(Hlength : forall la lb, length la = a -> length lb = b -> length (f la lb) = c)
(ta:tuple A a) (tb:tuple B b) : tuple C c