package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
type option_name = string list
type option_locality =
  1. | OptDefault
  2. | OptLocal
  3. | OptExport
  4. | OptGlobal
module MakeStringTable (A : sig ... end) : sig ... end
module MakeRefTable (A : sig ... end) : sig ... end
type !'a option_sig = {
  1. optdepr : bool;
  2. optname : string;
  3. optkey : option_name;
  4. optread : unit -> 'a;
  5. optwrite : 'a -> unit;
}
type !'a write_function = 'a -> unit
val declare_int_option : ?preprocess:(int option -> int option) -> int option option_sig -> int option write_function
val declare_bool_option : ?preprocess:(bool -> bool) -> bool option_sig -> bool write_function
val declare_string_option : ?preprocess:(string -> string) -> string option_sig -> string write_function
val declare_stringopt_option : ?preprocess:(string option -> string option) -> string option option_sig -> string option write_function
module OptionMap : sig ... end
val get_string_table : option_name -> < add : string -> unit ; mem : string -> unit ; print : unit ; remove : string -> unit >
val get_ref_table : option_name -> < add : Libnames.qualid -> unit ; mem : Libnames.qualid -> unit ; print : unit ; remove : Libnames.qualid -> unit >
val set_int_option_value_gen : ?locality:option_locality -> option_name -> int option -> unit
val set_bool_option_value_gen : ?locality:option_locality -> option_name -> bool -> unit
val set_string_option_value_gen : ?locality:option_locality -> option_name -> string -> unit
val set_string_option_append_value_gen : ?locality:option_locality -> option_name -> string -> unit
val unset_option_value_gen : ?locality:option_locality -> option_name -> unit
val set_int_option_value : option_name -> int option -> unit
val set_bool_option_value : option_name -> bool -> unit
val set_string_option_value : option_name -> string -> unit
val print_option_value : option_name -> unit
type option_value =
  1. | BoolValue of bool
  2. | IntValue of int option
  3. | StringValue of string
  4. | StringOptValue of string option
type option_state = {
  1. opt_depr : bool;
  2. opt_name : string;
  3. opt_value : option_value;
}
val get_tables : unit -> option_state OptionMap.t
val print_tables : unit -> Pp.t
val error_undeclared_key : option_name -> 'a