package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
exception End_of_input
val add : ontop:Stateid.t -> ?newtip:Stateid.t -> bool -> Vernacexpr.vernac_expr Loc.located -> Stateid.t * [ `NewTip | `Unfocus of Stateid.t ]
val query : at:Stateid.t -> route:Feedback.route_id -> Pcoq.Gram.coq_parsable -> unit
type focus = {
  1. start : Stateid.t;
  2. stop : Stateid.t;
  3. tip : Stateid.t;
}
val edit_at : Stateid.t -> [ `Focus of focus | `NewTip ]
val finish : unit -> unit
val observe : Stateid.t -> unit
val stop_worker : string -> unit
val join : unit -> unit
val snapshot_vio : Names.DirPath.t -> string -> unit
val reset_task_queue : unit -> unit
type tasks
val check_task : string -> tasks -> int -> bool
val info_tasks : tasks -> (string * float * int) list
val get_current_state : unit -> Stateid.t
val init : unit -> unit
val set_compilation_hints : string -> unit
val set_perspective : Stateid.t list -> unit
type document
val backup : unit -> document
val restore : document -> unit
type static_block_declaration = {
  1. block_start : Stateid.t;
  2. block_stop : Stateid.t;
  3. dynamic_switch : Stateid.t;
  4. carry_on_data : DynBlockData.t;
}
type document_node = {
  1. indentation : int;
  2. ast : Vernacexpr.vernac_expr;
  3. id : Stateid.t;
}
type document_view = {
  1. entry_point : document_node;
  2. prev_node : document_node -> document_node option;
}
type static_block_detection = document_view -> static_block_declaration option
type recovery_action = {
  1. base_state : Stateid.t;
  2. goals_to_admit : Goal.goal list;
  3. recovery_command : Vernacexpr.vernac_expr option;
}
type dynamic_block_error_recovery = static_block_declaration -> [ `Leaks | `ValidBlock of recovery_action ]
val register_proof_block_delimiter : Vernacexpr.proof_block_name -> static_block_detection -> dynamic_block_error_recovery -> unit
val state_computed_hook : (Stateid.t -> in_cache:bool -> unit) Hook.t
val unreachable_state_hook : (Stateid.t -> Exninfo.iexn -> unit) Hook.t
val state_ready_hook : (Stateid.t -> unit) Hook.t
val forward_feedback_hook : (Feedback.feedback -> unit) Hook.t
type state = {
  1. system : States.state;
  2. proof : Proof_global.state;
  3. shallow : bool;
}
val state_of_id : Stateid.t -> [ `Error of exn | `Expired | `Valid of state option ]
val current_proof_depth : unit -> int
val get_all_proof_names : unit -> Names.Id.t list
OCaml

Innovation. Community. Security.