package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
val safe_env : unit -> Safe_typing.safe_environment
val env : unit -> Environ.env
val env_is_initial : unit -> bool
val universes : unit -> UGraph.t
val named_context_val : unit -> Environ.named_context_val
val named_context : unit -> Context.Named.t
val set_engagement : Declarations.engagement -> unit
val set_typing_flags : Declarations.typing_flags -> unit
val push_named_assum : (Names.Id.t * Constr.types * bool) Univ.in_universe_context_set -> unit
val add_constraints : Univ.constraints -> unit
val push_context : bool -> Univ.universe_context -> unit
val push_context_set : bool -> Univ.universe_context_set -> unit
val start_module : Names.Id.t -> Names.module_path
val start_modtype : Names.Id.t -> Names.module_path
val exists_objlabel : Names.Label.t -> bool
val constant_of_delta_kn : Names.kernel_name -> Names.constant
val mind_of_delta_kn : Names.kernel_name -> Names.mutual_inductive
val opaque_tables : unit -> Opaqueproof.opaquetab
val body_of_constant : Names.constant -> Term.constr option
val body_of_constant_body : Declarations.constant_body -> Term.constr option
val global_universe_names : unit -> universe_names
val set_global_universe_names : universe_names -> unit
val start_library : Names.DirPath.t -> Names.module_path
val env_of_context : Environ.named_context_val -> Environ.env
val join_safe_environment : ?except:Future.UUIDSet.t -> unit -> unit
val is_joined_environment : unit -> bool
val is_polymorphic : Globnames.global_reference -> bool
val is_template_polymorphic : Globnames.global_reference -> bool
val is_type_in_type : Globnames.global_reference -> bool
val type_of_global_unsafe : Globnames.global_reference -> Constr.types
val register : Retroknowledge.field -> Term.constr -> Term.constr -> unit
val register_inline : Names.constant -> unit
val set_strategy : Names.constant Names.tableKey -> Conv_oracle.level -> unit
val current_dirpath : unit -> Names.dir_path
val with_global : (Environ.env -> Names.dir_path -> 'a Univ.in_universe_context_set) -> 'a
val global_env_summary_name : string
OCaml

Innovation. Community. Security.