diff options
| author | Maxime Dénès | 2017-06-14 18:16:31 +0200 |
|---|---|---|
| committer | Maxime Dénès | 2017-06-14 18:16:31 +0200 |
| commit | cb41d7b40c401c15e9cb66f508f89dbd1bdcdbff (patch) | |
| tree | f852248c2ce2be0cc3e6aae136e961561e395e85 /API | |
| parent | e70bec8fba8b15155aca41812225fcf42e1408e0 (diff) | |
| parent | f610068823b33bdc0af752a646df05b98489d7ce (diff) | |
Merge PR#763: [proof] Deprecate redundant wrappers.
Diffstat (limited to 'API')
| -rw-r--r-- | API/API.mli | 13 |
1 files changed, 11 insertions, 2 deletions
diff --git a/API/API.mli b/API/API.mli index 0cfa3e328d..68fbda7c73 100644 --- a/API/API.mli +++ b/API/API.mli @@ -3465,6 +3465,8 @@ sig (** @raise NoCurrentProof when outside proof mode. *) val discard_all : unit -> unit + val discard_current : unit -> unit + val get_current_proof_name : unit -> Names.Id.t end module Nametab : @@ -3940,11 +3942,18 @@ sig val solve : ?with_end_tac:unit Proofview.tactic -> Vernacexpr.goal_selector -> int option -> unit Proofview.tactic -> Proof.proof -> Proof.proof * bool - val delete_current_proof : unit -> unit val cook_proof : unit -> (Names.Id.t * (Safe_typing.private_constants Entries.definition_entry * Proof_global.proof_universes * Decl_kinds.goal_kind)) - val get_current_proof_name : unit -> Names.Id.t + val get_current_context : unit -> Evd.evar_map * Environ.env + + (* Deprecated *) + val delete_current_proof : unit -> unit + [@@ocaml.deprecated "use Proof_global.discard_current"] + + val get_current_proof_name : unit -> Names.Id.t + [@@ocaml.deprecated "use Proof_global.get_current_proof_name"] + end module Tactics : |
