aboutsummaryrefslogtreecommitdiff
path: root/src/Util/Tuple.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-11-06 17:10:45 -0500
committerGravatar Jason Gross <jgross@mit.edu>2016-11-06 17:10:45 -0500
commitbd28f5b205d54aa014587cbf03a322101fb0b021 (patch)
tree630e82fb1beb9f554ad9b7857947b57725e2e18e /src/Util/Tuple.v
parent7eed51d8ddd77fb6419be9fc6ff8450442322e57 (diff)
Add more admitted tuple lemmas
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 455c28f00..aca78cd5a 100644
--- a/src/Util/Tuple.v
+++ b/src/Util/Tuple.v
@@ -172,6 +172,11 @@ Lemma map_id {n A} (xs:tuple A n)
Proof.
Admitted.
+Lemma map_id_ext {n A} (f : A -> A) (xs:tuple A n)
+ : (forall x, f x = x) -> map f 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}