aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proof.ml
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-10-02 17:46:07 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-10-02 17:46:07 +0000
commit621625757d04bdb19075d92e764749d0a1393ce3 (patch)
treee04c688dbe4897de4781e68dec32fc92b92447a5 /proofs/proof.ml
parent8c24fc1ba49a1623dbecbea82c9fef238f17c4ee (diff)
Remove the unused "intel" field in Proof.proof_state
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15846 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs/proof.ml')
-rw-r--r--proofs/proof.ml15
1 files changed, 1 insertions, 14 deletions
diff --git a/proofs/proof.ml b/proofs/proof.ml
index 71afae020..bae5f1157 100644
--- a/proofs/proof.ml
+++ b/proofs/proof.ml
@@ -121,8 +121,6 @@ type proof_state = {
to unfocus the proof and the extra information stored while focusing.
The list is empty when the proof is fully unfocused. *)
focus_stack: (_focus_condition*focus_info*Proofview.focus_context) list;
- (* Extra information which can be freely used to create new behaviours. *)
- intel: Store.t
}
type proof_info = {
@@ -379,8 +377,7 @@ let unfocused = is_last_focus end_of_stack_kind
let start goals =
let pr =
{ state = { proofview = Proofview.init goals ;
- focus_stack = [] ;
- intel = Store.empty} ;
+ focus_stack = [] };
undo_stack = [] ;
transactions = [] ;
info = { endline_tactic = Proofview.tclUNIT ();
@@ -408,16 +405,6 @@ let return p =
unfocus end_of_stack_kind p;
Proofview.return p.state.proofview
-(*** Function manipulation proof extra informations ***)
-
-let get_proof_info pr =
- pr.state.intel
-
-let set_proof_info info pr =
- save pr;
- pr.state <- { pr.state with intel=info }
-
-
(*** Tactics ***)
let run_tactic env tac pr =