aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_3372.v
blob: eb70149a02309c1933bb95129c38976ad6b6b801 (plain)
1
2
3
4
5
6
7
8
Set Universe Polymorphism.
Definition hProp : Type := sigT (fun _ : Type => True).
Goal Type.
Fail exact hProp@{Set}. (* test that it fails, but is not an anomaly *)
try (exact hProp@{Set}; fail 1). (* Toplevel input, characters 15-32:
Anomaly: Uncaught exception Invalid_argument("Array.iter2", _).
Please report. *)
Abort.