(************************************************************************) (* v * The Coq Proof Assistant / The Coq Development Team *) (* glob_sign (** same as [fully_empty_glob_sign], but with [Global.env()] as environment *) (** Main globalization functions *) val glob_tactic : raw_tactic_expr -> glob_tactic_expr val glob_tactic_env : Id.t list -> Environ.env -> raw_tactic_expr -> glob_tactic_expr (** Low-level variants *) val intern_pure_tactic : glob_sign -> raw_tactic_expr -> glob_tactic_expr val intern_tactic_or_tacarg : glob_sign -> raw_tactic_expr -> Tacexpr.glob_tactic_expr val intern_constr : glob_sign -> constr_expr -> glob_constr_and_expr val intern_constr_with_bindings : glob_sign -> constr_expr * constr_expr bindings -> glob_constr_and_expr * glob_constr_and_expr bindings val intern_hyp : glob_sign -> Id.t Loc.located -> Id.t Loc.located (** Adds a globalization function for extra generic arguments *) val intern_genarg : glob_sign -> raw_generic_argument -> glob_generic_argument (** Adds a definition of tactics in the table *) val add_tacdef : Vernacexpr.locality_flag -> bool -> (Libnames.reference * bool * raw_tactic_expr) list -> unit val add_primitive_tactic : string -> glob_tactic_expr -> unit val lookup_ltacref : ltac_constant -> glob_tactic_expr (** printing *) val print_ltac : Libnames.qualid -> std_ppcmds (** Reduction expressions *) val intern_red_expr : glob_sign -> raw_red_expr -> glob_red_expr val dump_glob_red_expr : raw_red_expr -> unit (* Implemented in tacinterp *) val set_assert_tactic_installed : (string -> unit) -> unit