From 853821e4374050d5a770ee623b24a7bf15e288ae Mon Sep 17 00:00:00 2001 From: Jason Gross Date: Tue, 8 Nov 2016 11:22:11 -0500 Subject: Rename iffT, add some lemmas about tuple and hlist Some lemmas admitted --- src/Util/Tuple.v | 5 +++++ 1 file changed, 5 insertions(+) (limited to 'src/Util/Tuple.v') 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} -- cgit v1.2.3