package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
type t = private {
  1. prg_name : Names.Id.t;
  2. prg_body : Constr.constr;
  3. prg_type : Constr.constr;
  4. prg_ctx : UState.t;
  5. prg_univdecl : UState.universe_decl;
  6. prg_obligations : obligations;
  7. prg_deps : Names.Id.t list;
  8. prg_fixkind : fixpoint_kind option;
  9. prg_implicits : Impargs.manual_implicits;
  10. prg_notations : Vernacexpr.decl_notation list;
  11. prg_poly : bool;
  12. prg_scope : Declare.locality;
  13. prg_kind : Decls.definition_object_kind;
  14. prg_reduce : Constr.constr -> Constr.constr;
  15. prg_hook : Declare.Hook.t option;
  16. prg_opaque : bool;
}
val set_uctx : uctx:UState.t -> t -> t
OCaml

Innovation. Community. Security.