aboutsummaryrefslogtreecommitdiff
path: root/src/Util/Tuple.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-01-15 14:00:30 -0500
committerGravatar Jason Gross <jgross@mit.edu>2017-01-15 14:00:30 -0500
commit9e6105ece0d7c71c496752c8025b71732172f5e4 (patch)
treed4abedd0eb3bb028654977efe37535a33c91dd29 /src/Util/Tuple.v
parentd82f8f1c9543f4cdb637fc2735e65e77bfd0f0ad (diff)
Fix an issue with universes
We don't want to force the universe of [option] below other universes; to get template polymorphism to refresh universes, we need to eta-expand [option].
Diffstat (limited to 'src/Util/Tuple.v')
-rw-r--r--src/Util/Tuple.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/src/Util/Tuple.v b/src/Util/Tuple.v
index a5b299ac0..b97bfbc49 100644
--- a/src/Util/Tuple.v
+++ b/src/Util/Tuple.v
@@ -392,9 +392,9 @@ Local Notation option_bind
| None => None
end).
Definition lift_option {n A} (xs : tuple (option A) n) : option (tuple A n)
- := lift_monad option option_bind (@Some) xs.
+ := lift_monad (fun T => option T) option_bind (@Some) xs.
Definition push_option {n A} (xs : option (tuple A n)) : tuple (option A) n
- := push_monad option option_bind (@Some) xs.
+ := push_monad (fun T => option T) option_bind (@Some) xs.
Lemma lift_push_option {n A} (xs : option (tuple A (S n))) : lift_option (push_option xs) = xs.
Proof.