diff options
| author | Emilio Jesus Gallego Arias | 2020-04-02 01:08:24 -0400 |
|---|---|---|
| committer | Emilio Jesus Gallego Arias | 2020-04-15 11:07:18 -0400 |
| commit | 9908ce57e15a316ff692ce31f493651734998ded (patch) | |
| tree | 8f2a9571bb3a39607a8c17667789196d08fe1722 /doc/plugin_tutorial/tuto1/src | |
| parent | 35e363f988e941e710b4e24cd638233383275bd7 (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 'doc/plugin_tutorial/tuto1/src')
| -rw-r--r-- | doc/plugin_tutorial/tuto1/src/g_tuto1.mlg | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/doc/plugin_tutorial/tuto1/src/g_tuto1.mlg b/doc/plugin_tutorial/tuto1/src/g_tuto1.mlg index 73d94c2a51..8015d62eb4 100644 --- a/doc/plugin_tutorial/tuto1/src/g_tuto1.mlg +++ b/doc/plugin_tutorial/tuto1/src/g_tuto1.mlg @@ -286,7 +286,7 @@ END VERNAC COMMAND EXTEND ExploreProof CLASSIFIED AS QUERY | ![ proof_query ] [ "ExploreProof" ] -> { fun ~pstate -> - let sigma, env = Pfedit.get_current_context pstate in + let sigma, env = Proof_global.get_current_context pstate in let pprf = Proof.partial_proof (Proof_global.get_proof pstate) in Feedback.msg_notice (Pp.prlist_with_sep Pp.fnl (Printer.pr_econstr_env env sigma) pprf) |
