diff options
| author | Emilio Jesus Gallego Arias | 2020-01-30 23:36:19 +0100 |
|---|---|---|
| committer | Emilio Jesus Gallego Arias | 2020-01-30 23:36:19 +0100 |
| commit | 173a2d8b0fba1a85b618654151af04b5decf9bac (patch) | |
| tree | 8f7385dbc348bed11568414729ec4e1f65a295e4 /proofs/proof_bullet.ml | |
| parent | 869f731439b7fe034067bb550b60713b9b790f5b (diff) | |
[exn] Don't reraise in exception printers
This behaviour seems a bit dubious and it is indeed not needed, also
such re-raises seem like they will mess with the backtrace.
Diffstat (limited to 'proofs/proof_bullet.ml')
| -rw-r--r-- | proofs/proof_bullet.ml | 7 |
1 files changed, 3 insertions, 4 deletions
diff --git a/proofs/proof_bullet.ml b/proofs/proof_bullet.ml index 66e2ae5c29..61e8741973 100644 --- a/proofs/proof_bullet.ml +++ b/proofs/proof_bullet.ml @@ -79,7 +79,7 @@ module Strict = struct (function | FailedBullet (b,sugg) -> let prefix = Pp.(str"Wrong bullet " ++ pr_bullet b ++ str": ") in - CErrors.user_err ~hdr:"Focus" Pp.(prefix ++ suggest_on_error sugg) + Pp.(str "[Focus]" ++ spc () ++ prefix ++ suggest_on_error sugg) | _ -> raise CErrors.Unhandled) @@ -204,8 +204,7 @@ exception SuggestNoSuchGoals of int * Proof.t let _ = CErrors.register_handler begin function | SuggestNoSuchGoals(n,proof) -> let suffix = suggest proof in - CErrors.user_err - Pp.(str "No such " ++ str (CString.plural n "goal") ++ str "." ++ - pr_non_empty_arg (fun x -> x) suffix) + Pp.(str "No such " ++ str (CString.plural n "goal") ++ str "." ++ + pr_non_empty_arg (fun x -> x) suffix) | _ -> raise CErrors.Unhandled end |
