aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/polymorphism.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-07-07 17:04:45 +0200
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-07-07 17:06:39 +0200
commit7c7726a798caa6b506a727703de24d2bb5bb3956 (patch)
treee65226bba40098323b59cf8294cf12c1a5bffe82 /test-suite/success/polymorphism.v
parent024a7ab20b06d82571c68c3d2ac32cb60fb0053a (diff)
Univs: bug fix.
Missing universe substitutions of mind_params_ctxt when typechecking cases, which appeared only when let-ins were used.
Diffstat (limited to 'test-suite/success/polymorphism.v')
-rw-r--r--test-suite/success/polymorphism.v12
1 files changed, 12 insertions, 0 deletions
diff --git a/test-suite/success/polymorphism.v b/test-suite/success/polymorphism.v
index dc22b03f2..957612ef1 100644
--- a/test-suite/success/polymorphism.v
+++ b/test-suite/success/polymorphism.v
@@ -308,3 +308,15 @@ Definition RLRL' : forall x : R, RL x = RL (RL x).
Qed.
End eta.
+
+Module Hurkens'.
+ Require Import Hurkens.
+
+Polymorphic Record box (X : Type) (T := Type) : Type := wrap { unwrap : T }.
+
+Definition unwrap' := fun (X : Type) (b : box X) => let (unw) := b in unw.
+
+Fail Definition bad : False := TypeNeqSmallType.paradox (unwrap' Type (wrap _
+Type)) eq_refl.
+
+End Hurkens'. \ No newline at end of file