diff options
author | Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr> | 2014-09-29 11:00:48 +0200 |
---|---|---|
committer | Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr> | 2014-09-29 11:00:48 +0200 |
commit | f78bc2ca33c7bb7eb139e51c2cb74a3a63a040c9 (patch) | |
tree | 38b82efa66c449ebf7cea828582558f647544037 | |
parent | 2b3b6326c219984498f06707158a903307ff6795 (diff) |
Adding a test for bug #2428.
-rw-r--r-- | test-suite/bugs/2428.v | 10 |
1 files changed, 10 insertions, 0 deletions
diff --git a/test-suite/bugs/2428.v b/test-suite/bugs/2428.v new file mode 100644 index 000000000..a4f587a58 --- /dev/null +++ b/test-suite/bugs/2428.v @@ -0,0 +1,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. |