Module Ltac_plugin.Coretactics

val wit_hyp : (Names.lidentNames.lidentNames.Id.t) Genarg.genarg_type
val __coq_plugin_name : string
val delayed_list : ('a -> 'b -> 'b * 'c) list -> 'a -> 'b -> 'b * 'c list
val simple_induct : Tactypes.quantified_hypothesis -> unit Proofview.tactic
val simple_destruct : Tactypes.quantified_hypothesis -> unit Proofview.tactic
val initial_atomic : unit -> unit
val initial_name : string -> Tacexpr.ml_tactic_name
val initial_entry : string -> Tacexpr.ml_tactic_entry
val register_list_tactical : string -> (unit Proofview.tactic list -> unit Proofview.tactic) -> unit
val initial_tacticals : unit -> unit