From 43fa7ce9a96617aa777ef8ea15f133d80131fcad Mon Sep 17 00:00:00 2001 From: Jason Gross Date: Wed, 6 Jun 2018 12:42:38 -0400 Subject: 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. --- src/Util/CPSNotations.v | 1 + 1 file changed, 1 insertion(+) (limited to 'src/Util/CPSNotations.v') 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]. *) -- cgit v1.2.3