summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/5065.v
blob: 932fee8b3b4302d096be46b807887717822e3921 (plain)
1
2
3
4
5
6
Inductive foo := C1 : bar -> foo with bar := C2 : foo -> bar.

Lemma L1 : foo -> True with L2 : bar -> True.
intros; clear L1 L2; abstract (exact I).
intros; exact I.
Qed.