aboutsummaryrefslogtreecommitdiff
path: root/vernac/vernacstate.mli
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2020-04-02 01:41:20 -0400
committerEmilio Jesus Gallego Arias2020-04-15 11:12:10 -0400
commit0c748e670ef1a81cb35c1cc55892dba141c25930 (patch)
treed90cc4362019557a74d6d1ac46701e0d6178e8ce /vernac/vernacstate.mli
parent9908ce57e15a316ff692ce31f493651734998ded (diff)
[proof] Merge `Proof_global` into `Declare`
We place creation and saving of interactive proofs in the same module; this will allow to make `proof_entry` private, improving invariants and control over clients, and to reduce the API [for example next commit will move abstract declaration into this module, removing the exported ad-hoc `build_constant_by_tactic`] Next step will be to unify all the common code in the interactive / non-interactive case; but we need to tweak the handling of obligations first.
Diffstat (limited to 'vernac/vernacstate.mli')
-rw-r--r--vernac/vernacstate.mli18
1 files changed, 9 insertions, 9 deletions
diff --git a/vernac/vernacstate.mli b/vernac/vernacstate.mli
index 9c4de7720c..2cabbe35f5 100644
--- a/vernac/vernacstate.mli
+++ b/vernac/vernacstate.mli
@@ -25,8 +25,8 @@ module LemmaStack : sig
val pop : t -> Lemmas.t * t option
val push : t option -> Lemmas.t -> t
- val map_top_pstate : f:(Proof_global.t -> Proof_global.t) -> t -> t
- val with_top_pstate : t -> f:(Proof_global.t -> 'a ) -> 'a
+ val map_top_pstate : f:(Declare.t -> Declare.t) -> t -> t
+ val with_top_pstate : t -> f:(Declare.t -> 'a ) -> 'a
end
@@ -50,7 +50,7 @@ val make_shallow : t -> t
val invalidate_cache : unit -> unit
(* Compatibility module: Do Not Use *)
-module Proof_global : sig
+module Declare : sig
exception NoCurrentProof
@@ -65,16 +65,16 @@ module Proof_global : sig
val with_current_proof :
(unit Proofview.tactic -> Proof.t -> Proof.t * 'a) -> 'a
- val return_proof : unit -> Proof_global.closed_proof_output
- val return_partial_proof : unit -> Proof_global.closed_proof_output
+ val return_proof : unit -> Declare.closed_proof_output
+ val return_partial_proof : unit -> Declare.closed_proof_output
- type closed_proof = Proof_global.proof_object * Lemmas.Info.t
+ type closed_proof = Declare.proof_object * Lemmas.Info.t
val close_future_proof :
feedback_id:Stateid.t ->
- Proof_global.closed_proof_output Future.computation -> closed_proof
+ Declare.closed_proof_output Future.computation -> closed_proof
- val close_proof : opaque:Proof_global.opacity_flag -> keep_body_ucst_separate:bool -> closed_proof
+ val close_proof : opaque:Declare.opacity_flag -> keep_body_ucst_separate:bool -> closed_proof
val discard_all : unit -> unit
val update_global_env : unit -> unit
@@ -89,7 +89,7 @@ module Proof_global : sig
val get : unit -> LemmaStack.t option
val set : LemmaStack.t option -> unit
- val get_pstate : unit -> Proof_global.t option
+ val get_pstate : unit -> Declare.t option
val freeze : marshallable:bool -> LemmaStack.t option
val unfreeze : LemmaStack.t -> unit