package coq
type cl_typ =
| CL_SORT
| CL_FUN
| CL_SECVAR of Names.variable
| CL_CONST of Names.constant
| CL_IND of Names.inductive
| CL_PROJ of Names.constant
val subst_cl_typ : Mod_subst.substitution -> cl_typ -> cl_typ
type coe_typ = Globnames.global_reference
type inheritance_path = coe_index list
val class_exists : cl_typ -> bool
val class_info : cl_typ -> cl_index * cl_info_typ
val class_info_from_index : cl_index -> cl_typ * cl_info_typ
val find_class_type :
Evd.evar_map ->
EConstr.types ->
cl_typ * EConstr.EInstance.t * EConstr.constr list
val class_of :
Environ.env ->
Evd.evar_map ->
EConstr.types ->
EConstr.types * cl_index
val inductive_class_of : Names.inductive -> cl_index
val class_args_of :
Environ.env ->
Evd.evar_map ->
EConstr.types ->
EConstr.constr list
val coercion_exists : coe_typ -> bool
val coercion_value :
coe_index ->
(EConstr.unsafe_judgment * bool * bool) Univ.in_universe_context_set
val lookup_path_between_class : (cl_index * cl_index) -> inheritance_path
val lookup_path_between :
Environ.env ->
Evd.evar_map ->
(EConstr.types * EConstr.types) ->
EConstr.types * EConstr.types * inheritance_path
val lookup_path_to_fun_from :
Environ.env ->
Evd.evar_map ->
EConstr.types ->
EConstr.types * inheritance_path
val lookup_path_to_sort_from :
Environ.env ->
Evd.evar_map ->
EConstr.types ->
EConstr.types * inheritance_path
val lookup_pattern_path_between :
Environ.env ->
(Names.inductive * Names.inductive) ->
(Names.constructor * int) list
val install_path_printer :
(((cl_index * cl_index) * inheritance_path) -> Pp.std_ppcmds) ->
unit
val string_of_class : cl_typ -> string
val pr_class : cl_typ -> Pp.std_ppcmds
val pr_cl_index : cl_index -> Pp.std_ppcmds
val inheritance_graph : unit -> ((cl_index * cl_index) * inheritance_path) list
val classes : unit -> cl_typ list
val coercions : unit -> coe_index list
val hide_coercion : coe_typ -> int option
sectionYPositions = computeSectionYPositions($el), 10)"
x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
>