val __coq_plugin_name : stringval pr_fun_ind_using : 'a -> 'b -> ('a -> 'b -> 'c -> Pp.t) -> ('a -> 'b -> 'c -> Pp.t) -> 'd -> ('c * 'c Tactypes.bindings) option -> Pp.tval pr_fun_ind_using_typed : (Environ.env -> Evd.evar_map -> 'a -> Pp.t) -> (Environ.env -> Evd.evar_map -> 'a -> Pp.t) -> 'b -> (Environ.env -> Evd.evar_map -> 'c * ('a * 'a Tactypes.bindings)) option -> Pp.tval wit_fun_ind_using : (Constrexpr.constr_expr Tactypes.with_bindings option, Genintern.glob_constr_and_expr Tactypes.with_bindings option, EConstr.constr Tactypes.with_bindings Tactypes.delayed_open option) Genarg.genarg_typeval fun_ind_using : Constrexpr.constr_expr Tactypes.with_bindings option Pcoq.Entry.tval pr_intro_as_pat : 'a -> 'b -> 'c -> 'd option -> Pp.tval out_disjunctive : Tactypes.delayed_open_constr Tactypes.intro_pattern_expr CAst.t -> Tactypes.delayed_open_constr Tactypes.or_and_intro_pattern_expr CAst.tval wit_with_names : (Constrexpr.constr_expr Tactypes.intro_pattern_expr CAst.t option, Genintern.glob_constr_and_expr Tactypes.intro_pattern_expr CAst.t option, Ltac_plugin.Tacexpr.intro_pattern option) Genarg.genarg_typeval with_names : Constrexpr.constr_expr Tactypes.intro_pattern_expr CAst.t option Pcoq.Entry.tval functional_induction : 'a -> EConstr.constr -> (EConstr.constr * EConstr.constr Tactypes.bindings) option -> Tactypes.delayed_open_constr Tactypes.intro_pattern_expr CAst.t option -> unit Proofview.tacticval pr_constr_comma_sequence : 'a -> 'b -> ('a -> 'b -> 'c -> Pp.t) -> 'd -> 'e -> 'c list -> Pp.tval wit_constr_comma_sequence' : (Constrexpr.constr_expr list, Genintern.glob_constr_and_expr list, EConstr.constr list) Genarg.genarg_typeval constr_comma_sequence' : Constrexpr.constr_expr list Pcoq.Entry.tval pr_auto_using : 'a -> 'b -> ('a -> 'b -> 'c -> Pp.t) -> 'd -> 'e -> 'c list -> Pp.tval wit_auto_using' : (Constrexpr.constr_expr list, Genintern.glob_constr_and_expr list, EConstr.constr list) Genarg.genarg_typeval auto_using' : Constrexpr.constr_expr list Pcoq.Entry.t
val wit_function_fix_definition : Vernacexpr.fixpoint_expr Loc.located Genarg.uniform_genarg_typeval function_fix_definition : Vernacexpr.fixpoint_expr Loc.located Pcoq.Entry.tval is_proof_termination_interactively_checked : ('a * Constrexpr.recursion_order_expr_r CAst.t option Vernacexpr.fix_expr_gen) list -> boolval classify_as_Fixpoint : ('a * Vernacexpr.fixpoint_expr) list -> Vernacextend.vernac_classificationval classify_funind : ('a * Vernacexpr.fixpoint_expr) list -> Vernacextend.vernac_classificationval is_interactive : ('a * Vernacexpr.fixpoint_expr) list -> boolval pr_fun_scheme_arg : (Names.Id.t * Libnames.qualid * Sorts.family) -> Pp.tval wit_fun_scheme_arg : (Names.Id.t * Libnames.qualid * Sorts.family, unit, unit) Genarg.genarg_typeval fun_scheme_arg : (Names.Id.t * Libnames.qualid * Sorts.family) Pcoq.Entry.tval warning_error : Libnames.qualid list -> exn -> unit