summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/5065.v
blob: 6bd677ba6f55e85234df2de11b042a1b95fc2816 (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.