aboutsummaryrefslogtreecommitdiff
path: root/src/Util/CPSNotations.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jagro@google.com>2018-06-06 12:42:38 -0400
committerGravatar Jason Gross <jasongross9@gmail.com>2018-06-14 16:37:49 -0400
commit43fa7ce9a96617aa777ef8ea15f133d80131fcad (patch)
tree71ffabafd3a6379e6463dd0f9eb828cbd390a416 /src/Util/CPSNotations.v
parentedc8f44af48b8bde22750af3ab3b2f855bbdb6f9 (diff)
Set universe polymorphism in CPSNotations
This bypasses universe inconsistencies that arise when trying to return continuations from other continuations, which is a scenario that comes up frequently with cpsbind.
Diffstat (limited to 'src/Util/CPSNotations.v')
-rw-r--r--src/Util/CPSNotations.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/src/Util/CPSNotations.v b/src/Util/CPSNotations.v
index 0f49176c5..87e46e41c 100644
--- a/src/Util/CPSNotations.v
+++ b/src/Util/CPSNotations.v
@@ -1,4 +1,5 @@
Require Import Crypto.Util.Notations.
+Local Set Universe Polymorphism.
(** [x <- f ; C] encodes a call to function [f] with [C] as the
continuation. In [C], [x] refers to the output of [f]. *)