aboutsummaryrefslogtreecommitdiff
path: root/toplevel/coqloop.ml
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2020-04-02 01:08:24 -0400
committerEmilio Jesus Gallego Arias2020-04-15 11:07:18 -0400
commit9908ce57e15a316ff692ce31f493651734998ded (patch)
tree8f2a9571bb3a39607a8c17667789196d08fe1722 /toplevel/coqloop.ml
parent35e363f988e941e710b4e24cd638233383275bd7 (diff)
[proof] Move proof_global functionality to Proof_global from Pfedit
This actually gets `Pfedit` out of the dependency picture [can be almost merged with `Proof` now, as it is what it manipulates] and would allow to reduce the exported low-level API from `Proof_global`, as `map_fold_proof` is not used anymore.
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 b8acdd3af1..ff33663926 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 = Pfedit.get_proof_context p in
+ let sigma, env = Proof_global.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
- | Pfedit.NoSuchGoal
+ | Proof_global.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
- | Pfedit.NoSuchGoal
+ | Proof_global.NoSuchGoal
| Option.IsNone ->
CErrors.user_err (str "No goals to show.")