package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
type 'a declaration_hook
val set_start_hook : (EConstr.types -> unit) -> unit
val start_proof_com : ?inference_hook:Pretyping.inference_hook -> Decl_kinds.goal_kind -> Vernacexpr.proof_expr list -> unit declaration_hook -> unit
val start_proof_with_initialization : Decl_kinds.goal_kind -> Evd.evar_map -> (bool * Proof_global.lemma_possible_guards * unit Proofview.tactic list option) option -> ((Names.Id.t * Proof_global.universe_binders option) * (Term.types * (Names.Name.t list * Impargs.manual_explicitation list))) list -> int list option -> unit declaration_hook -> unit
val set_save_hook : (Proof.proof -> unit) -> unit
val save_proof : ?proof:Proof_global.closed_proof -> Vernacexpr.proof_end -> unit
val get_current_context : unit -> Evd.evar_map * Environ.env
OCaml

Innovation. Community. Security.