aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/pattern.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-01-04 14:06:05 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-01-04 14:06:05 +0000
commitc7f63628e3659cc95235c71402c43b50aef3893d (patch)
treed2211ac6efb49e0aa5eba20b4ea4b17d0f63e693 /test-suite/success/pattern.v
parentf3979966ec7d1e5c13fd77e2d19856a3dd2e7a3f (diff)
Errors issued by reduction tactics (e.g. pattern) were not caught by "try".
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12621 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/pattern.v')
-rw-r--r--test-suite/success/pattern.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/test-suite/success/pattern.v b/test-suite/success/pattern.v
index 23e6f8e35..72f84052d 100644
--- a/test-suite/success/pattern.v
+++ b/test-suite/success/pattern.v
@@ -42,3 +42,8 @@ Goal 0=1->1=0->True.
intros H1 H2.
pattern 0 at 1, 1 in H1, H2 || exact I. (* check pattern fails *)
Qed.
+
+(* Test catching of reduction tactics errors (was not the case in 8.2) *)
+Goal eq_refl 0 = eq_refl 0.
+pattern 0 at 1 || reflexivity.
+Qed.