summaryrefslogtreecommitdiff
path: root/test-suite/misc/poly-capture-global-univs/theories/evil.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/misc/poly-capture-global-univs/theories/evil.v')
-rw-r--r--test-suite/misc/poly-capture-global-univs/theories/evil.v13
1 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/misc/poly-capture-global-univs/theories/evil.v b/test-suite/misc/poly-capture-global-univs/theories/evil.v
new file mode 100644
index 00000000..7fd98c27
--- /dev/null
+++ b/test-suite/misc/poly-capture-global-univs/theories/evil.v
@@ -0,0 +1,13 @@
+
+Declare ML Module "evil_plugin".
+
+Evil T f. (* <- if this doesn't fail then the rest goes through *)
+
+Definition g : Type -> Set := f.
+
+Require Import Hurkens.
+
+Lemma absurd : False.
+Proof.
+ exact (TypeNeqSmallType.paradox (g Type) eq_refl).
+Qed.