diff options
| author | Emilio Jesus Gallego Arias | 2020-05-20 00:37:35 +0200 |
|---|---|---|
| committer | Emilio Jesus Gallego Arias | 2020-06-26 14:38:10 +0200 |
| commit | 7d183d8a12a03a608a3dc8a724142468b45886ac (patch) | |
| tree | e95ba16a3f6c9b84c18a54f1f88ecd5bb5bff227 /vernac/declare.mli | |
| parent | 1f121ebf2990dc25899f2f3eb138eddd147483cf (diff) | |
[declare] Make ProgramDecl.t abstract
This hides even more internals; we will reduce the API even more
shortly.
Diffstat (limited to 'vernac/declare.mli')
| -rw-r--r-- | vernac/declare.mli | 17 |
1 files changed, 5 insertions, 12 deletions
diff --git a/vernac/declare.mli b/vernac/declare.mli index 30db26e693..6f104e764d 100644 --- a/vernac/declare.mli +++ b/vernac/declare.mli @@ -462,18 +462,7 @@ type fixpoint_kind = IsFixpoint of lident option list | IsCoFixpoint (* Information about a single [Program {Definition,Lemma,..}] declaration *) module ProgramDecl : sig - type t = private - { prg_name : Id.t - ; prg_info : CInfo.t - ; prg_body : constr - ; prg_type : constr - ; prg_uctx : UState.t - ; prg_obligations : obligations - ; prg_deps : Id.t list - ; prg_fixkind : fixpoint_kind option - ; prg_notations : Vernacexpr.decl_notation list - ; prg_reduce : constr -> constr - } + type t val make : Names.Id.t @@ -488,12 +477,16 @@ module ProgramDecl : sig -> RetrieveObl.obligation_info -> t + val show : t -> Pp.t + (* This is internal, only here as obligations get merged into the regular declaration path *) module Internal : sig val get_poly : t -> bool + val get_name : t -> Id.t val get_uctx : t -> UState.t val set_uctx : uctx:UState.t -> t -> t + val get_obligations : t -> obligations end end |
