package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
val async_proofs_worker_id : string Stdlib.ref
val async_proofs_is_worker : unit -> bool
val load_vos_libraries : bool Stdlib.ref
val debug : bool Stdlib.ref
val in_debugger : bool Stdlib.ref
val in_toplevel : bool Stdlib.ref
val profile : bool
val we_are_parsing : bool Stdlib.ref
val raw_print : bool Stdlib.ref
val beautify : bool Stdlib.ref
val beautify_file : bool Stdlib.ref
val quiet : bool Stdlib.ref
val silently : ('a -> 'b) -> 'a -> 'b
val verbosely : ('a -> 'b) -> 'a -> 'b
val if_silent : ('a -> unit) -> 'a -> unit
val if_verbose : ('a -> unit) -> 'a -> unit
val warn : bool Stdlib.ref
val make_warn : bool -> unit
val if_warn : ('a -> unit) -> 'a -> unit
val with_modified_ref : 'c Stdlib.ref -> ('c -> 'c) -> ('a -> 'b) -> 'a -> 'b
val with_option : bool Stdlib.ref -> ('a -> 'b) -> 'a -> 'b
val with_options : bool Stdlib.ref list -> ('a -> 'b) -> 'a -> 'b
val without_option : bool Stdlib.ref -> ('a -> 'b) -> 'a -> 'b
val with_extra_values : 'c list Stdlib.ref -> 'c list -> ('a -> 'b) -> 'a -> 'b
val get_native_compiler : unit -> bool
val set_native_compiler : bool -> unit
val set_inline_level : int -> unit
val get_inline_level : unit -> int
val default_inline_level : int
val profile_ltac : bool Stdlib.ref
val profile_ltac_cutoff : float Stdlib.ref
OCaml

Innovation. Community. Security.