aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/pfedit.mli
diff options
context:
space:
mode:
authorGravatar gareuselesinge <gareuselesinge@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-10-18 13:52:15 +0000
committerGravatar gareuselesinge <gareuselesinge@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-10-18 13:52:15 +0000
commit168424263f9c8510a4c51d59a2945babd20880f4 (patch)
tree8afc3396e03d0568506470b639d2a2d1ba897fa1 /proofs/pfedit.mli
parent020aa7a8e9bca88631e6d7fa68d1ff462f5af25a (diff)
declaration_hooks use Ephemeron
Ideally, any component of the global state that is a function or any other unmarshallable data should be stocked as an ephemeron to make the state always marshallable. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16893 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs/pfedit.mli')
-rw-r--r--proofs/pfedit.mli8
1 files changed, 4 insertions, 4 deletions
diff --git a/proofs/pfedit.mli b/proofs/pfedit.mli
index 79929fd8d..7df0da800 100644
--- a/proofs/pfedit.mli
+++ b/proofs/pfedit.mli
@@ -75,15 +75,15 @@ val cook_this_proof : (Proof.proof -> unit) ->
(Entries.definition_entry list *
lemma_possible_guards *
Decl_kinds.goal_kind *
- unit Tacexpr.declaration_hook) ->
+ unit Tacexpr.declaration_hook Ephemeron.key) ->
Id.t *
(Entries.definition_entry * lemma_possible_guards * goal_kind *
- unit declaration_hook)
+ unit declaration_hook Ephemeron.key)
val cook_proof : (Proof.proof -> unit) ->
Id.t *
(Entries.definition_entry * lemma_possible_guards * goal_kind *
- unit declaration_hook)
+ unit declaration_hook Ephemeron.key)
(** {6 ... } *)
(** [get_pftreestate ()] returns the current focused pending proof.
@@ -104,7 +104,7 @@ val get_current_goal_context : unit -> Evd.evar_map * env
(** [current_proof_statement] *)
val current_proof_statement :
- unit -> Id.t * goal_kind * types * unit declaration_hook
+ unit -> Id.t * goal_kind * types * unit declaration_hook Ephemeron.key
(** {6 ... } *)
(** [get_current_proof_name ()] return the name of the current focused