aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--proofs/logic.ml2
-rw-r--r--test-suite/success/pattern.v5
2 files changed, 7 insertions, 0 deletions
diff --git a/proofs/logic.ml b/proofs/logic.ml
index 0fbd8ad21..f0f03febb 100644
--- a/proofs/logic.ml
+++ b/proofs/logic.ml
@@ -53,6 +53,8 @@ let rec catchable_exception = function
| Util.UserError _ | TypeError _
| RefinerError _ | Indrec.RecursionSchemeError _
| Nametab.GlobalizationError _ | PretypeError (_,VarNotFound _)
+ (* reduction errors *)
+ | Tacred.ReductionTacticError _
(* unification errors *)
| PretypeError(_,(CannotUnify _|CannotUnifyLocal _|CannotGeneralize _
|NoOccurrenceFound _|CannotUnifyBindingType _|NotClean _
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.