aboutsummaryrefslogtreecommitdiff
path: root/src/Util/Tuple.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-11-06 17:09:45 -0500
committerGravatar Jason Gross <jgross@mit.edu>2016-11-06 17:09:45 -0500
commit7eed51d8ddd77fb6419be9fc6ff8450442322e57 (patch)
treecfbeadc5333cf3da816a4dbaed1866aef259dd36 /src/Util/Tuple.v
parent12d083871316497a1743b0fbac14514d39996aeb (diff)
Add more admitted tuple lemmas
Diffstat (limited to 'src/Util/Tuple.v')
-rw-r--r--src/Util/Tuple.v15
1 files changed, 15 insertions, 0 deletions
diff --git a/src/Util/Tuple.v b/src/Util/Tuple.v
index 554f9e14e..455c28f00 100644
--- a/src/Util/Tuple.v
+++ b/src/Util/Tuple.v
@@ -157,6 +157,21 @@ Lemma map_map2 {n A B C D} (f:A -> B -> C) (g:C -> D) (xs:tuple A n) (ys:tuple B
Proof.
Admitted.
+Lemma map2_fst {n A B C} (f:A -> C) (xs:tuple A n) (ys:tuple B n)
+ : map2 (fun a b => f a) xs ys = map f xs.
+Proof.
+Admitted.
+
+Lemma map2_snd {n A B C} (f:B -> C) (xs:tuple A n) (ys:tuple B n)
+ : map2 (fun a b => f b) xs ys = map f ys.
+Proof.
+Admitted.
+
+Lemma map_id {n A} (xs:tuple A n)
+ : map (fun x => x) xs = 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}