aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2015-02-26 17:22:41 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2015-02-26 17:22:41 +0100
commitbc7d29e4c0f53d5c8e654157c4137c7e82910a7a (patch)
tree72ddb080c47bfc2462148c992fe4968991789586 /test-suite
parent31846ce3bb4053a4fd121afd6aa8260b0c5dff18 (diff)
Test for bug #3298.
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/bugs/closed/3298.v (renamed from test-suite/bugs/opened/3298.v)6
1 files changed, 2 insertions, 4 deletions
diff --git a/test-suite/bugs/opened/3298.v b/test-suite/bugs/closed/3298.v
index bce7c3f23..3a7de4567 100644
--- a/test-suite/bugs/opened/3298.v
+++ b/test-suite/bugs/closed/3298.v
@@ -4,8 +4,7 @@ Module JGross.
Goal forall H : False, match H return Set with end.
Proof.
intros.
- Fail solve [ eauto ]. (* No applicable tactic *)
- admit.
+ solve [ eauto ].
Qed.
End JGross.
@@ -17,7 +16,6 @@ Section BenDelaware.
Qed.
Goal forall (H : False), match H return Set with end.
Proof.
- Fail solve [ eauto ] .
- admit.
+ solve [ eauto ] .
Qed.
End BenDelaware.