aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/Tactics.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-03-12 13:18:42 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-05-17 23:38:26 +0200
commit741f3fab052b91eaec57f32b639ca722c3d8dc34 (patch)
tree3beff509deee6f7220017ca8d67eec3ee479210e /test-suite/output/Tactics.v
parent6d770156669dd9868ae7623b8f4302866e2cc8c7 (diff)
A fix for #5390 (a useful error on used introduction names was masked).
With the "apply in" introduction pattern, and the backtrack possibly done in "apply" over the components of conjunctions (descend_in_conjunctions), the reasons for failing might have different sources. We give priority to the detection of used names over other (unification) errors so that an error there is not masked in the backtracking made by descend_in_conjunctions. Of course, the question of what best unification error to give in the presence of backtracking is still open.
Diffstat (limited to 'test-suite/output/Tactics.v')
-rw-r--r--test-suite/output/Tactics.v10
1 files changed, 10 insertions, 0 deletions
diff --git a/test-suite/output/Tactics.v b/test-suite/output/Tactics.v
index a7c497cfa..9a5edb813 100644
--- a/test-suite/output/Tactics.v
+++ b/test-suite/output/Tactics.v
@@ -11,3 +11,13 @@ Print Ltac f.
Ltac g := match goal with |- context [if ?X then _ else _ ] => case X end.
Print Ltac g.
+
+(* Test an error message (#5390) *)
+Lemma myid (P : Prop) : P <-> P.
+Proof. split; auto. Qed.
+
+Goal True -> (True /\ True) -> True.
+Proof.
+intros H.
+Fail intros [H%myid ?].
+Fail destruct 1 as [H%myid ?].