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 /plugins | |
| 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 'plugins')
| -rw-r--r-- | plugins/extraction/extract_env.ml | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/plugins/extraction/extract_env.ml b/plugins/extraction/extract_env.ml index 3a90d24c97..40dbf8bea4 100644 --- a/plugins/extraction/extract_env.ml +++ b/plugins/extraction/extract_env.ml @@ -729,7 +729,7 @@ let extract_and_compile l = let show_extraction ~pstate = init ~inner:true false false; let prf = Proof_global.get_proof pstate in - let sigma, env = Pfedit.get_current_context pstate in + let sigma, env = Proof_global.get_current_context pstate in let trms = Proof.partial_proof prf in let extr_term t = let ast, ty = extract_constr env sigma t in |
