aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/vernacentries.mli
diff options
context:
space:
mode:
Diffstat (limited to 'toplevel/vernacentries.mli')
-rw-r--r--toplevel/vernacentries.mli5
1 files changed, 3 insertions, 2 deletions
diff --git a/toplevel/vernacentries.mli b/toplevel/vernacentries.mli
index 0eca1143f..2e6e35df4 100644
--- a/toplevel/vernacentries.mli
+++ b/toplevel/vernacentries.mli
@@ -13,6 +13,7 @@ open Names
open Term
open Vernacinterp
open Vernacexpr
+open Topconstr
(*i*)
(* Vernacular entries. This module registers almost all the vernacular entries,
@@ -52,9 +53,9 @@ type pcoq_hook = {
solve : int -> unit;
abort : string -> unit;
search : searchable -> dir_path list * bool -> unit;
- print_name : Libnames.qualid Util.located -> unit;
+ print_name : Libnames.reference -> unit;
print_check : Environ.unsafe_judgment -> unit;
- print_eval : (constr -> constr) -> Environ.env -> Coqast.t -> Environ.unsafe_judgment -> unit;
+ print_eval : (constr -> constr) -> Environ.env -> constr_expr -> Environ.unsafe_judgment -> unit;
show_goal : int option -> unit
}