aboutsummaryrefslogtreecommitdiff
path: root/src/Util/CPSNotations.v
diff options
context:
space:
mode:
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]. *)