package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
val register_ltac : Vernacexpr.locality_flag -> ?deprecation:Vernacinterp.deprecation -> Tacexpr.tacdef_body list -> unit
type !'a grammar_tactic_prod_item_expr = 'a Pptactic.grammar_tactic_prod_item_expr =
  1. | TacTerm of string
  2. | TacNonTerm of ('a * Names.Id.t option) Loc.located
type raw_argument = string * string option
val register_tactic_notation_entry : string -> ('a, 'b, 'c) Genarg.genarg_type -> unit
val add_ml_tactic_notation : Tacexpr.ml_tactic_name -> level:int -> ?deprecation:Vernacinterp.deprecation -> argument grammar_tactic_prod_item_expr list list -> unit
val create_ltac_quotation : string -> ('grm Loc.located -> Tacexpr.raw_tactic_arg) -> ('grm Pcoq.Entry.t * int option) -> unit
val print_ltacs : unit -> unit
val print_located_tactic : Libnames.qualid -> unit
type !_ ty_sig =
  1. | TyNil : (Geninterp.interp_sign -> unit Proofview.tactic) ty_sig
  2. | TyIdent : string * 'r ty_sig -> 'r ty_sig
  3. | TyArg : ('a, 'b, 'c) Extend.ty_user_symbol * string * 'r0 ty_sig -> ('c -> 'r0) ty_sig
  4. | TyAnonArg : ('a0, 'b0, 'c0) Extend.ty_user_symbol * 'r1 ty_sig -> 'r1 ty_sig
type ty_ml =
  1. | TyML : 'r ty_sig * 'r -> ty_ml
val tactic_extend : string -> string -> level:Int.t -> ?deprecation:Vernacinterp.deprecation -> ty_ml list -> unit
OCaml

Innovation. Community. Security.