package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
type vodigest =
  1. | Dvo_or_vi of Digest.t
  2. | Dvivo of Digest.t * Digest.t
val digest_match : actual:vodigest -> required:vodigest -> bool
type safe_environment
val empty_environment : safe_environment
val is_initial : safe_environment -> bool
val env_of_safe_env : safe_environment -> Environ.env
type safe_transformer0 = safe_environment -> safe_environment
type !'a safe_transformer = safe_environment -> 'a * safe_environment
type private_constant
type private_constants
type private_constant_role =
  1. | Subproof
  2. | Schema of Names.inductive * string
val side_effects_of_private_constants : private_constants -> Entries.side_effect list
val empty_private_constants : private_constants
val private_con_of_con : safe_environment -> Names.constant -> private_constant
val private_con_of_scheme : kind:string -> safe_environment -> (Names.inductive * Names.constant) list -> private_constant
val inline_private_constants_in_constr : Environ.env -> Constr.constr -> private_constants -> Constr.constr
val universes_of_private : private_constants -> Univ.universe_context_set list
val is_curmod_library : safe_environment -> bool
val join_safe_environment : ?except:Future.UUIDSet.t -> safe_environment -> safe_environment
val is_joined_environment : safe_environment -> bool
type global_declaration =
  1. | ConstantEntry of bool * private_constants Entries.constant_entry
  2. | GlobalRecipe of Cooking.recipe
val push_context_set : bool -> Univ.universe_context_set -> safe_transformer0
val push_context : bool -> Univ.universe_context -> safe_transformer0
val add_constraints : Univ.constraints -> safe_transformer0
val current_modpath : safe_environment -> Names.module_path
val current_dirpath : safe_environment -> Names.dir_path
type compiled_library
type native_library = Nativecode.global list
val get_library_native_symbols : safe_environment -> Names.DirPath.t -> Nativecode.symbols
type judgment
val j_val : judgment -> Term.constr
val j_type : judgment -> Term.constr
val exists_objlabel : Names.Label.t -> safe_environment -> bool
val retroknowledge : (Retroknowledge.retroknowledge -> 'a) -> safe_environment -> 'a
val register_inline : Names.constant -> safe_transformer0
OCaml

Innovation. Community. Security.