aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/refiner.ml
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-02-18 19:45:36 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-02-18 19:45:36 +0000
commit4c1ccb9e2a4b219ac5180115bc4267e1b059cdd1 (patch)
tree9ecfc27037e02802b1e6884517ca930cb8197cbc /proofs/refiner.ml
parentb101df5536146b9c3cd3569fc3b6334650f2a300 (diff)
Removing Exc_located and using the new exception enrichement
mechanism to retrieve the same information. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16215 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs/refiner.ml')
-rw-r--r--proofs/refiner.ml10
1 files changed, 5 insertions, 5 deletions
diff --git a/proofs/refiner.ml b/proofs/refiner.ml
index 332f255b2..4592c60dd 100644
--- a/proofs/refiner.ml
+++ b/proofs/refiner.ml
@@ -216,15 +216,15 @@ let tclSHOWHYPS (tac : tactic) (goal: Goal.goal Evd.sigma)
let catch_failerror e =
if catchable_exception e then check_for_interrupt ()
else match e with
- | FailError (0,_) | Loc.Exc_located(_, FailError (0,_))
+ | FailError (0,_)
| LtacLocated (_,_,FailError (0,_)) ->
check_for_interrupt ()
- | FailError (lvl,s) -> raise (FailError (lvl - 1, s))
- | Loc.Exc_located(s,FailError (lvl,s')) ->
- raise (Loc.Exc_located(s,FailError (lvl - 1, s')))
+ | FailError (lvl,s) ->
+ raise (Exninfo.copy e (FailError (lvl - 1, s)))
| LtacLocated (s'',loc,FailError (lvl,s')) ->
raise (LtacLocated (s'',loc,FailError (lvl - 1,s')))
| e -> raise e
+ (** FIXME: do we need to add a [Errors.push] here? *)
(* ORELSE0 t1 t2 tries to apply t1 and if it fails, applies t2 *)
let tclORELSE0 t1 t2 g =
@@ -325,7 +325,7 @@ let tclTIMEOUT n t g =
restore_timeout ();
res
with
- | TacTimeout | Loc.Exc_located(_,TacTimeout) ->
+ | TacTimeout ->
restore_timeout ();
errorlabstrm "Refiner.tclTIMEOUT" (str"Timeout!")
| e -> restore_timeout (); raise e