summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/7392.v
blob: cf465c658857a03367ba5f2a058a009ed9f29859 (plain)
1
2
3
4
5
6
7
8
9
Inductive R : nat -> Prop := ER : forall n, R n -> R (S n).

Goal (forall (n : nat), R n -> False) -> True -> False.
Proof.
intros H0 H1.
eapply H0.
clear H1.
apply ER.
simpl.