aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-05-28 19:18:07 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-05-28 19:18:07 +0000
commit7edfbedba1426282b69b7bc8bc01259015c27e0a (patch)
tree514b62a01523b48360d5a6ce53b9031d789587fd /proofs
parent10b68837fd896663cfb908228000732903471db6 (diff)
Getting rid of LtacLocated exception transformer.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16535 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs')
-rw-r--r--proofs/logic.ml1
-rw-r--r--proofs/proof_type.ml3
-rw-r--r--proofs/proof_type.mli7
-rw-r--r--proofs/proofview.ml1
-rw-r--r--proofs/refiner.ml5
5 files changed, 5 insertions, 12 deletions
diff --git a/proofs/logic.ml b/proofs/logic.ml
index a0781ae6a..7dc3fb49a 100644
--- a/proofs/logic.ml
+++ b/proofs/logic.ml
@@ -57,7 +57,6 @@ let is_unification_error = function
| _ -> false
let rec catchable_exception = function
- | LtacLocated(_,_,e) -> catchable_exception e
| Errors.UserError _ | TypeError _
| RefinerError _ | Indrec.RecursionSchemeError _
| Nametab.GlobalizationError _
diff --git a/proofs/proof_type.ml b/proofs/proof_type.ml
index 954e2fdb7..f7f10272c 100644
--- a/proofs/proof_type.ml
+++ b/proofs/proof_type.ml
@@ -58,5 +58,4 @@ type ltac_call_kind =
type ltac_trace = (int * Loc.t * ltac_call_kind) list
-exception LtacLocated of ltac_trace * Loc.t * exn
-
+let (ltac_trace_info : (ltac_trace * Loc.t) Exninfo.t) = Exninfo.make ()
diff --git a/proofs/proof_type.mli b/proofs/proof_type.mli
index 33945052f..74a12d42b 100644
--- a/proofs/proof_type.mli
+++ b/proofs/proof_type.mli
@@ -73,6 +73,8 @@ type tactic = goal sigma -> goal list sigma
(** Ltac traces *)
+(** TODO: Move those definitions somewhere sensible *)
+
type ltac_call_kind =
| LtacNotationCall of string
| LtacNameCall of ltac_constant
@@ -83,7 +85,4 @@ type ltac_call_kind =
type ltac_trace = (int * Loc.t * ltac_call_kind) list
-(** Invariant: the exceptions embedded in LtacLocated satisfy
- Errors.noncritical *)
-
-exception LtacLocated of ltac_trace * Loc.t * exn
+val ltac_trace_info : (ltac_trace * Loc.t) Exninfo.t
diff --git a/proofs/proofview.ml b/proofs/proofview.ml
index 1066c173b..96ff63d23 100644
--- a/proofs/proofview.ml
+++ b/proofs/proofview.ml
@@ -334,7 +334,6 @@ let tclEXTEND tacs1 rtac tacs2 env =
this should be maintained synchronized, probably. *)
open Pretype_errors
let rec catchable_exception = function
- | Proof_type.LtacLocated(_,_,e) -> catchable_exception e
| Errors.UserError _
| Type_errors.TypeError _ | PretypeError (_,_,TypingError _)
| Indrec.RecursionSchemeError _
diff --git a/proofs/refiner.ml b/proofs/refiner.ml
index 5a71b6816..dfc9c0a63 100644
--- a/proofs/refiner.ml
+++ b/proofs/refiner.ml
@@ -216,13 +216,10 @@ 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,_)
- | LtacLocated (_,_,FailError (0,_)) ->
+ | FailError (0,_) ->
check_for_interrupt ()
| 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? *)