package coq
module Id : sig ... end
module Name : sig ... end
type variable = Id.t
type module_ident = Id.t
module ModIdset : sig ... end
module ModIdmap : sig ... end
module DirPath : sig ... end
module Label : sig ... end
module MBId : sig ... end
module MBIset : sig ... end
module MBImap : sig ... end
module ModPath : sig ... end
module MPset : sig ... end
module MPmap : sig ... end
module KerName : sig ... end
module KNset : sig ... end
module KNpred : sig ... end
module KNmap : sig ... end
module Constant : sig ... end
module Cpred : sig ... end
module Cset : sig ... end
module Cset_env : sig ... end
module Cmap : sig ... end
module Cmap_env : sig ... end
module MutInd : sig ... end
module Mindset : sig ... end
module Mindmap : sig ... end
module Mindmap_env : sig ... end
type inductive = MutInd.t * int
type constructor = inductive * int
module Indmap : sig ... end
module Constrmap : sig ... end
module Indmap_env : sig ... end
module Constrmap_env : sig ... end
val constr_modpath : constructor -> ModPath.t
val ith_constructor_of_inductive : inductive -> int -> constructor
val inductive_of_constructor : constructor -> inductive
val index_of_constructor : constructor -> int
val ind_hash : inductive -> int
val ind_user_hash : inductive -> int
val ind_syntactic_hash : inductive -> int
val eq_constructor : constructor -> constructor -> bool
val eq_user_constructor : constructor -> constructor -> bool
val eq_syntactic_constructor : constructor -> constructor -> bool
val constructor_ord : constructor -> constructor -> int
val constructor_hash : constructor -> int
val constructor_user_ord : constructor -> constructor -> int
val constructor_user_hash : constructor -> int
val constructor_syntactic_ord : constructor -> constructor -> int
val constructor_syntactic_hash : constructor -> int
type global_reference =
| VarRef of variable
| ConstRef of Constant.t
| IndRef of inductive
| ConstructRef of constructor
val eq_egr : evaluable_global_reference -> evaluable_global_reference -> bool
val hcons_con : Constant.t -> Constant.t
val hcons_construct : constructor -> constructor
val empty_transparent_state : transparent_state
val full_transparent_state : transparent_state
val var_full_transparent_state : transparent_state
val cst_full_transparent_state : transparent_state
val eq_constant_key : Constant.t -> Constant.t -> bool
val eq_con_chk : Constant.t -> Constant.t -> bool
type identifier = Id.t
val string_of_id : Id.t -> string
val id_of_string : string -> Id.t
module Idset : sig ... end
module Idpred : sig ... end
module Idmap : sig ... end
type dir_path = DirPath.t
val make_dirpath : module_ident list -> DirPath.t
val repr_dirpath : DirPath.t -> module_ident list
val empty_dirpath : DirPath.t
val is_empty_dirpath : DirPath.t -> bool
val string_of_dirpath : DirPath.t -> string
val initial_dir : DirPath.t
type label = Label.t
val mk_label : string -> Label.t
val string_of_label : Label.t -> string
type mod_bound_id = MBId.t
val string_of_mbid : MBId.t -> string
val debug_string_of_mbid : MBId.t -> string
type module_path = ModPath.t =
val check_bound_mp : ModPath.t -> bool
val string_of_mp : ModPath.t -> string
val initial_path : ModPath.t
type kernel_name = KerName.t
val string_of_kn : KerName.t -> string
type constant = Constant.t
module Projection : sig ... end
type projection = Projection.t
val constant_of_kn_equiv : KerName.t -> KerName.t -> Constant.t
val constant_of_kn : KerName.t -> Constant.t
val make_con : ModPath.t -> DirPath.t -> Label.t -> Constant.t
val repr_con : Constant.t -> ModPath.t * DirPath.t * Label.t
val user_con : Constant.t -> KerName.t
val canonical_con : Constant.t -> KerName.t
val con_modpath : Constant.t -> ModPath.t
val con_label : Constant.t -> Label.t
val eq_constant : Constant.t -> Constant.t -> bool
val con_ord : Constant.t -> Constant.t -> int
val con_user_ord : Constant.t -> Constant.t -> int
val con_with_label : Constant.t -> Label.t -> Constant.t
val string_of_con : Constant.t -> string
val pr_con : Constant.t -> Pp.t
val debug_pr_con : Constant.t -> Pp.t
val debug_string_of_con : Constant.t -> string
type mutual_inductive = MutInd.t
val string_of_mind : MutInd.t -> string
val debug_string_of_mind : MutInd.t -> string
sectionYPositions = computeSectionYPositions($el), 10)"
x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
>