aboutsummaryrefslogtreecommitdiffhomepage
path: root/API
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2017-11-21 13:56:15 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2017-11-21 13:56:15 +0100
commit0e01de69c22a3793855b4c97c50e4514191b19bc (patch)
tree446a0ec91c87746f946fb9352aa23fafd2b8c7f3 /API
parent74e60947d78e3610312aa1702f12143841c5a7cf (diff)
parent8cada511701d8893bab5553470ab721b33713043 (diff)
Merge PR #6181: [proof] Attempt to deprecate some V82 parts of the proof API.
Diffstat (limited to 'API')
-rw-r--r--API/API.mli7
1 files changed, 7 insertions, 0 deletions
diff --git a/API/API.mli b/API/API.mli
index 8a4a6cc89..cc0de2b1b 100644
--- a/API/API.mli
+++ b/API/API.mli
@@ -4645,16 +4645,23 @@ sig
type proof
type 'a focus_kind
+ val proof : proof ->
+ Goal.goal list * (Goal.goal list * Goal.goal list) list *
+ Goal.goal list * Goal.goal list * Evd.evar_map
+
val run_tactic : Environ.env ->
unit Proofview.tactic -> proof -> proof * (bool * Proofview_monad.Info.tree)
val unshelve : proof -> proof
val maximal_unfocus : 'a focus_kind -> proof -> proof
val pr_proof : proof -> Pp.t
+
module V82 :
sig
val grab_evars : proof -> proof
val subgoals : proof -> Goal.goal list Evd.sigma
+ [@@ocaml.deprecated "Use the first and fifth argument of [Proof.proof]"]
+
end
end