aboutsummaryrefslogtreecommitdiff
path: root/toplevel/coqloop.ml
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2020-04-11 17:19:12 -0400
committerEmilio Jesus Gallego Arias2020-04-15 11:12:43 -0400
commite262a6262ebb6c3010cb58e96839b0e3d66e09ac (patch)
tree478ded36ca29b20b41119759bbf1a03827c9dfb8 /toplevel/coqloop.ml
parent28fc9aff20c39a04ad0e58e1bb8ec52c13631b61 (diff)
[proof] Move functions related to `Proof.t` to `Proof`
This makes the API more orthogonal and allows better structure in future code.
Diffstat (limited to 'toplevel/coqloop.ml')
-rw-r--r--toplevel/coqloop.ml6
1 files changed, 3 insertions, 3 deletions
diff --git a/toplevel/coqloop.ml b/toplevel/coqloop.ml
index 86fd3be4f5..2c5faa4df7 100644
--- a/toplevel/coqloop.ml
+++ b/toplevel/coqloop.ml
@@ -375,7 +375,7 @@ let exit_on_error =
point we should consolidate the code *)
let show_proof_diff_to_pp pstate =
let p = Option.get pstate in
- let sigma, env = Declare.get_proof_context p in
+ let sigma, env = Proof.get_proof_context p in
let pprf = Proof.partial_proof p in
Pp.prlist_with_sep Pp.fnl (Printer.pr_econstr_env env sigma) pprf
@@ -392,7 +392,7 @@ let show_proof_diff_cmd ~state removed =
let show_removed = Some removed in
Pp_diff.diff_pp_combined ~tokenize_string ?show_removed o_pp n_pp
with
- | Declare.NoSuchGoal
+ | Proof.NoSuchGoal _
| Option.IsNone -> n_pp
| Pp_diff.Diff_Failure msg -> begin
(* todo: print the unparsable string (if we know it) *)
@@ -403,7 +403,7 @@ let show_proof_diff_cmd ~state removed =
else
n_pp
with
- | Declare.NoSuchGoal
+ | Proof.NoSuchGoal _
| Option.IsNone ->
CErrors.user_err (str "No goals to show.")