aboutsummaryrefslogtreecommitdiff
path: root/proofs
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2019-06-09 14:20:17 +0200
committerPierre-Marie Pédrot2019-06-09 14:20:17 +0200
commit1f81679d117446d32fcad8012e5613cb2377b359 (patch)
tree216bcc16b1cfce4d2a6ce1ce4356f3a5a7fffd0d /proofs
parent73c2dc60ccd4d64506250a9c7476740e97ab022c (diff)
parent1c52097ecfccd22b7515f0e197b747107874b372 (diff)
Merge PR #8726: More robust treatment of the Discharge status
Reviewed-by: aspiwack Ack-by: ejgallego Reviewed-by: ppedrot
Diffstat (limited to 'proofs')
-rw-r--r--proofs/pfedit.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/proofs/pfedit.ml b/proofs/pfedit.ml
index 66b47a64a7..c7fcc66120 100644
--- a/proofs/pfedit.ml
+++ b/proofs/pfedit.ml
@@ -117,7 +117,7 @@ open Decl_kinds
let next = let n = ref 0 in fun () -> incr n; !n
-let build_constant_by_tactic id ctx sign ?(goal_kind = Global, false, Proof Theorem) typ tac =
+let build_constant_by_tactic id ctx sign ?(goal_kind = Global ImportDefaultBehavior, false, Proof Theorem) typ tac =
let evd = Evd.from_ctx ctx in
let terminator = Proof_global.make_terminator (fun _ -> ()) in
let goals = [ (Global.env_of_context sign , typ) ] in
@@ -139,7 +139,7 @@ let build_constant_by_tactic id ctx sign ?(goal_kind = Global, false, Proof Theo
let build_by_tactic ?(side_eff=true) env sigma ?(poly=false) typ tac =
let id = Id.of_string ("temporary_proof"^string_of_int (next())) in
let sign = val_of_named_context (named_context env) in
- let gk = Global, poly, Proof Theorem in
+ let gk = Global ImportDefaultBehavior, poly, Proof Theorem in
let ce, status, univs =
build_constant_by_tactic id sigma sign ~goal_kind:gk typ tac in
let body = Future.force ce.const_entry_body in