aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel
diff options
context:
space:
mode:
Diffstat (limited to 'toplevel')
-rw-r--r--toplevel/obligations.mli4
-rw-r--r--toplevel/vernacentries.ml5
2 files changed, 5 insertions, 4 deletions
diff --git a/toplevel/obligations.mli b/toplevel/obligations.mli
index 69d206961..80b689144 100644
--- a/toplevel/obligations.mli
+++ b/toplevel/obligations.mli
@@ -87,9 +87,9 @@ val add_mutual_definitions :
fixpoint_kind -> unit
val obligation : int * Names.Id.t option * Constrexpr.constr_expr option ->
- Tacexpr.raw_tactic_expr option -> unit
+ Genarg.glob_generic_argument option -> unit
-val next_obligation : Names.Id.t option -> Tacexpr.raw_tactic_expr option -> unit
+val next_obligation : Names.Id.t option -> Genarg.glob_generic_argument option -> unit
val solve_obligations : Names.Id.t option -> unit Proofview.tactic option -> progress
(* Number of remaining obligations to be solved for this program *)
diff --git a/toplevel/vernacentries.ml b/toplevel/vernacentries.ml
index c1142c7cb..eff4d15c0 100644
--- a/toplevel/vernacentries.ml
+++ b/toplevel/vernacentries.ml
@@ -844,8 +844,9 @@ let focus_command_cond = Proof.no_cond command_focus
let vernac_solve_existential = instantiate_nth_evar_com
let vernac_set_end_tac tac =
- (** FIXME *)
- let tac = Genarg.out_gen (Genarg.rawwit Constrarg.wit_ltac) tac in
+ let open Genintern in
+ let env = { genv = Global.env (); ltacvars = Id.Set.empty } in
+ let _, tac = Genintern.generic_intern env tac in
if not (refining ()) then
error "Unknown command of the non proof-editing mode.";
set_end_tac tac