Module Section
val depth : 'a t -> int
Number of nested sections (0 if no sections are open)
Manipulating sections
type section_entry
=
|
SecDefinition of Names.Constant.t
|
SecInductive of Names.MutInd.t
val open_section : custom:'a -> 'a t -> 'a t
Open a new section with the provided universe polymorphic status. Sections can be nested, with the proviso that polymorphic sections cannot appear inside a monomorphic one. A custom data can be attached to this section, that will be returned by
close_section
.
val close_section : 'a t -> 'a t * section_entry list * Univ.ContextSet.t * 'a
Close the current section and returns the entries defined inside, the set of global monomorphic constraints added in this section, and the custom data provided at the opening of the section.
Extending sections
val push_context : (Names.Name.t array * Univ.UContext.t) -> 'a t -> 'a t
Extend the current section with a local universe context. Assumes that the last opened section is polymorphic.
val push_constraints : Univ.ContextSet.t -> 'a t -> 'a t
Extend the current section with a global universe context. Assumes that the last opened section is monomorphic.
val push_constant : poly:bool -> Names.Constant.t -> 'a t -> 'a t
Make the constant as having been defined in this section.
val push_inductive : poly:bool -> Names.MutInd.t -> 'a t -> 'a t
Make the inductive block as having been defined in this section.
Retrieving section data
type abstr_info
= private
{
abstr_ctx : Constr.named_context;
Section variables of this prefix
abstr_subst : Univ.Instance.t;
Actual names of the abstracted variables
abstr_uctx : Univ.AUContext.t;
Universe quantification, same length as the substitution
}
Data needed to abstract over the section variable and universe hypotheses
val empty_segment : abstr_info
Nothing to abstract
val segment_of_constant : Environ.env -> Names.Constant.t -> 'a t -> abstr_info
Section segment at the time of the constant declaration
val segment_of_inductive : Environ.env -> Names.MutInd.t -> 'a t -> abstr_info
Section segment at the time of the inductive declaration
val replacement_context : Environ.env -> 'a t -> Opaqueproof.work_list
Section segments of all declarations from this section.
val is_in_section : Environ.env -> Names.GlobRef.t -> 'a t -> bool