aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proof_global.mli
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-11-09 19:44:17 +0100
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-11-09 19:44:17 +0100
commitce80fa3cb3e6d8809bb3ee015bff39c67c0aed16 (patch)
treebe80159f44855799c885174910de3931fdde07b2 /proofs/proof_global.mli
parent91c2a866e7827c0ede0539cb49f924b68db569a9 (diff)
new: Optimize Proof, Optimize Heap
- drops all Defined entries from the evar map (applying the subst to the initial evar and the undefined evars types). - call Gc.compact Now the question is: where should these two commands be documented?
Diffstat (limited to 'proofs/proof_global.mli')
-rw-r--r--proofs/proof_global.mli2
1 files changed, 2 insertions, 0 deletions
diff --git a/proofs/proof_global.mli b/proofs/proof_global.mli
index de259a4cc..8dd739686 100644
--- a/proofs/proof_global.mli
+++ b/proofs/proof_global.mli
@@ -46,6 +46,8 @@ exception NoCurrentProof
val give_me_the_proof : unit -> Proof.proof
(** @raise NoCurrentProof when outside proof mode. *)
+val compact_the_proof : unit -> unit
+
(** When a proof is closed, it is reified into a [proof_object], where
[id] is the name of the proof, [entries] the list of the proof terms
(in a form suitable for definitions). Together with the [terminator]