summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/5641.v
blob: 9f3246f33da093db01cc3344826239eed8e395c0 (plain)
1
2
3
4
5
6
Set Universe Polymorphism.

Definition foo@{i j} (A : Type@{i}) : Type@{j}.
Proof.
abstract (exact ltac:(abstract (exact A))).
Defined.