diff options
| author | Emilio Jesus Gallego Arias | 2019-02-14 13:10:08 +0100 |
|---|---|---|
| committer | Gaƫtan Gilbert | 2019-04-24 14:01:11 +0200 |
| commit | ed1b663afdd02355877c51dc9c759ddfd91b0854 (patch) | |
| tree | fe94e5bebe4455ad7dbf613d03fc9ca1385ce940 /engine/proofview.ml | |
| parent | 75c5264aa687480c66a6765d64246b5ebd2c0d54 (diff) | |
[proof] Fix proof bullet error helper which was implemented as a hook
We add the information on the proper layer by catching the low-level
exception.
Diffstat (limited to 'engine/proofview.ml')
| -rw-r--r-- | engine/proofview.ml | 17 |
1 files changed, 3 insertions, 14 deletions
diff --git a/engine/proofview.ml b/engine/proofview.ml index 316f02bc37..86dcb8ab3b 100644 --- a/engine/proofview.ml +++ b/engine/proofview.ml @@ -345,22 +345,11 @@ let tclBREAK = Proof.break exception NoSuchGoals of int -(* This hook returns a string to be appended to the usual message. - Primarily used to add a suggestion about the right bullet to use to - focus the next goal, if applicable. *) -let nosuchgoals_hook:(int -> Pp.t) ref = ref (fun n -> mt ()) -let set_nosuchgoals_hook f = nosuchgoals_hook := f - - - -(* This uses the hook above *) let _ = CErrors.register_handler begin function | NoSuchGoals n -> - let suffix = !nosuchgoals_hook n in - CErrors.user_err - (str "No such " ++ str (String.plural n "goal") ++ str "." ++ - pr_non_empty_arg (fun x -> x) suffix) - | _ -> raise CErrors.Unhandled + CErrors.user_err + (str "No such " ++ str (String.plural n "goal") ++ str ".") + | _ -> raise CErrors.Unhandled end (** [tclFOCUS_gen nosuchgoal i j t] applies [t] in a context where |
