package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
type !'a proof_entry = private {
  1. proof_entry_body : 'a Entries.const_entry_body;
  2. proof_entry_secctx : Names.Id.Set.t option;
  3. proof_entry_feedback : Stateid.t option;
  4. proof_entry_type : Constr.types option;
  5. proof_entry_universes : Entries.universes_entry;
  6. proof_entry_opaque : bool;
  7. proof_entry_inline_code : bool;
}
type variable_declaration =
  1. | SectionLocalDef of Evd.side_effects proof_entry
  2. | SectionLocalAssum of {
    1. typ : Constr.types;
    2. impl : Glob_term.binding_kind;
    }
type !'a constant_entry =
  1. | DefinitionEntry of 'a proof_entry
  2. | ParameterEntry of Entries.parameter_entry
  3. | PrimitiveEntry of Entries.primitive_entry
val declare_universe_context : poly:bool -> Univ.ContextSet.t -> unit
val declare_variable : name:Names.variable -> kind:Decls.logical_kind -> variable_declaration -> unit
val definition_entry : ?fix_exn:Future.fix_exn -> ?opaque:bool -> ?inline:bool -> ?types:Constr.types -> ?univs:Entries.universes_entry -> ?eff:Evd.side_effects -> Constr.constr -> Evd.side_effects proof_entry
val pure_definition_entry : ?fix_exn:Future.fix_exn -> ?opaque:bool -> ?inline:bool -> ?types:Constr.types -> ?univs:Entries.universes_entry -> Constr.constr -> unit proof_entry
val delayed_definition_entry : ?opaque:bool -> ?inline:bool -> ?feedback_id:Stateid.t -> ?section_vars:Names.Id.Set.t -> ?univs:Entries.universes_entry -> ?types:Constr.types -> 'a Entries.const_entry_body -> 'a proof_entry
type import_status =
  1. | ImportDefaultBehavior
  2. | ImportNeedQualified
val declare_private_constant : ?role:Evd.side_effect_role -> ?local:import_status -> name:Names.Id.t -> kind:Decls.logical_kind -> unit proof_entry -> Names.Constant.t * Evd.side_effects
val inline_private_constants : univs:UState.t -> Environ.env -> Evd.side_effects proof_entry -> Constr.t * UState.t
val definition_message : Names.Id.t -> unit
val assumption_message : Names.Id.t -> unit
val fixpoint_message : int array option -> Names.Id.t list -> unit
val cofixpoint_message : Names.Id.t list -> unit
val recursive_message : bool -> int array option -> Names.Id.t list -> unit
val check_exists : Names.Id.t -> unit
exception AlreadyDeclared of string option * Names.Id.t
module Internal : sig ... end
OCaml

Innovation. Community. Security.