aboutsummaryrefslogtreecommitdiff
path: root/src/Util/Tuple.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-11-08 11:22:11 -0500
committerGravatar Jason Gross <jgross@mit.edu>2016-11-08 11:22:11 -0500
commit853821e4374050d5a770ee623b24a7bf15e288ae (patch)
treecec7afb052b974bc081618ae5ab5a4275800cd30 /src/Util/Tuple.v
parentf929cd20f82206be0bdf40b91c179dcb346408e1 (diff)
Rename iffT, add some lemmas about tuple and hlist
Some lemmas admitted
Diffstat (limited to 'src/Util/Tuple.v')
-rw-r--r--src/Util/Tuple.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/src/Util/Tuple.v b/src/Util/Tuple.v
index 21abfed3a..4d97c7857 100644
--- a/src/Util/Tuple.v
+++ b/src/Util/Tuple.v
@@ -193,6 +193,11 @@ Lemma map_id_ext {n A} (f : A -> A) (xs:tuple A n)
Proof.
Admitted.
+Lemma map_map {n A B C} (g : B -> C) (f : A -> B) (xs:tuple A n)
+ : map g (map f xs) = map (fun x => g (f x)) xs.
+Proof.
+Admitted.
+
Section monad.
Context (M : Type -> Type) (bind : forall X Y, M X -> (X -> M Y) -> M Y) (ret : forall X, X -> M X).
Fixpoint lift_monad' {n A} {struct n}