aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_2428.v
blob: b398a76d91555525368c5ca7c1d49bdb56cff53e (plain)
1
2
3
4
5
6
7
8
9
10
Axiom P : nat -> Prop.

Definition myFact := forall x, P x.

Hint Extern 1 (P _) => progress (unfold myFact in *).

Lemma test : (True -> myFact) -> P 3.
Proof.
  intros. debug eauto.
Qed.