aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs
diff options
context:
space:
mode:
Diffstat (limited to 'proofs')
-rw-r--r--proofs/pfedit.ml2
-rw-r--r--proofs/proof_global.ml10
2 files changed, 5 insertions, 7 deletions
diff --git a/proofs/pfedit.ml b/proofs/pfedit.ml
index e953d2074..fff1a121d 100644
--- a/proofs/pfedit.ml
+++ b/proofs/pfedit.ml
@@ -151,7 +151,7 @@ open Decl_kinds
let next = let n = ref 0 in fun () -> incr n; !n
let build_constant_by_tactic id sign typ tac =
- start_proof id (Global,false,Proof Theorem) sign typ (fun _ _ -> ());
+ start_proof id (Global,Proof Theorem) sign typ (fun _ _ -> ());
try
by tac;
let _,(const,_,_,_) = cook_proof (fun _ -> ()) in
diff --git a/proofs/proof_global.ml b/proofs/proof_global.ml
index fa108f1ec..bcd9d6e0d 100644
--- a/proofs/proof_global.ml
+++ b/proofs/proof_global.ml
@@ -265,18 +265,16 @@ let close_proof () =
let id = get_current_proof_name () in
let p = give_me_the_proof () in
let proofs_and_types = Proof.return p in
- let { compute_guard=cg ; strength=str ; hook=hook } =
- Idmap.find id !proof_info
- in
- let (_, poly, _) = str in
let entries = List.map
(fun (c,t) -> { Entries.const_entry_body = c ;
const_entry_type = Some t;
- const_entry_polymorphic = poly;
const_entry_opaque = true })
proofs_and_types
in
- (id,(entries,cg,str,hook))
+ let { compute_guard=cg ; strength=str ; hook=hook } =
+ Idmap.find id !proof_info
+ in
+ (id, (entries,cg,str,hook))
with
| Proof.UnfinishedProof ->
Util.error "Attempt to save an incomplete proof"