aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/omega
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-04-07 16:31:25 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-04-07 17:23:50 +0200
commit2ba1351849550c50e0fe2c7fc7f63758c10fb14a (patch)
treef4f3673d2650ff97418aa56b8ac912db0c51b576 /plugins/omega
parent3a1df73d60372d1966c69450f80a66ca72cb9b44 (diff)
Fix an unhandled exception in Omega.
Diffstat (limited to 'plugins/omega')
-rw-r--r--plugins/omega/coq_omega.ml1
1 files changed, 1 insertions, 0 deletions
diff --git a/plugins/omega/coq_omega.ml b/plugins/omega/coq_omega.ml
index a2016cb03..7780de712 100644
--- a/plugins/omega/coq_omega.ml
+++ b/plugins/omega/coq_omega.ml
@@ -1884,6 +1884,7 @@ let destructure_goal =
(mkApp (Lazy.force coq_dec_not_not, [| t; dec; mkNewMeta () |]))))
intro
with Undecidable -> Tactics.elim_type (Lazy.force coq_False)
+ | e when Proofview.V82.catchable_exception e -> Proofview.tclZERO e
in
Tacticals.New.tclTHEN goal_tac destructure_hyps
in