aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-07-10 15:59:44 +0200
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-07-11 10:15:06 +0200
commit2a805fd99b96746dbfe381d64cd7eaba84fdca79 (patch)
tree77e0c47e097c4edebe9eea5f839488c91264e9b3 /proofs
parent31b99c5671c956de455372e43f935e1c70006f9d (diff)
Feedback: LoadedFile + Goals
LoadedFile is generated when a .vo is loaded Goals is generated when -feedback-goals
Diffstat (limited to 'proofs')
-rw-r--r--proofs/proof_global.ml1
-rw-r--r--proofs/proof_global.mli1
2 files changed, 2 insertions, 0 deletions
diff --git a/proofs/proof_global.ml b/proofs/proof_global.ml
index 06afc2fa9..7c7ff0c94 100644
--- a/proofs/proof_global.ml
+++ b/proofs/proof_global.ml
@@ -515,4 +515,5 @@ let freeze ~marshallable =
| `Shallow -> !pstates
| `No -> !pstates
let unfreeze s = pstates := s; update_proof_mode ()
+let proof_of_state = function { proof }::_ -> proof | _ -> raise NoCurrentProof
diff --git a/proofs/proof_global.mli b/proofs/proof_global.mli
index d5229c562..2b54b24ef 100644
--- a/proofs/proof_global.mli
+++ b/proofs/proof_global.mli
@@ -188,3 +188,4 @@ end
type state
val freeze : marshallable:[`Yes | `No | `Shallow] -> state
val unfreeze : state -> unit
+val proof_of_state : state -> Proof.proof