coq-core.kernel
Names.Constant
btauto_plugin
cc_plugin
coq-core.clib
coq-core.config
coq-core.engine
coq-core.gramlib
coq-core.interp
coq-core.lib
coq-core.library
coq-core.parsing
coq-core.plugins
coq-core.pretyping
coq-core.printing
coq-core.proofs
coq-core.stm
coq-core.sysinit
coq-core.tactics
coq-core.top_printers
coq-core.toplevel
coq-core.vernac
coq-core.vm
coqide-server.core
coqide-server.protocol
derive_plugin
extraction_plugin
firstorder_plugin
float_syntax_plugin
funind_plugin
ltac2_plugin
ltac_plugin
micromega_plugin
nsatz_plugin
number_string_notation_plugin
ring_plugin
rtauto_plugin
ssreflect_plugin
ssrmatching_plugin
ssrsearch_plugin
tauto_plugin
tuto0_plugin
tuto1_plugin
tuto2_plugin
tuto3_plugin
zify_plugin
type t
Constructors
val make : KerName.t -> KerName.t -> t
Builds a constant name from a user and a canonical kernel name.
val make1 : KerName.t -> t
Special case of make where the user name is canonical.
make
val make2 : ModPath.t -> Label.t -> t
Shortcut for (make1 (KerName.make2 ...))
(make1 (KerName.make2 ...))
Projections
val user : t -> KerName.t
val canonical : t -> KerName.t
val repr2 : t -> ModPath.t * Label.t
Shortcut for KerName.repr (user ...)
KerName.repr (user ...)
val modpath : t -> ModPath.t
Shortcut for KerName.modpath (user ...)
KerName.modpath (user ...)
val label : t -> Label.t
Shortcut for KerName.label (user ...)
KerName.label (user ...)
Comparisons
include QNameS with type t := t
module CanOrd : EqType with type t = t
Equality functions over the canonical name. Their use should be restricted to the kernel.
module UserOrd : EqType with type t = t
Equality functions over the user name.
module SyntacticOrd : EqType with type t = t
Equality functions using both names, for low-level uses.
val equal : t -> t -> bool
Default comparison, alias for CanOrd.equal
CanOrd.equal
val hash : t -> int
Hashing function
val change_label : t -> Label.t -> t
Builds a new constant name with a different label
Displaying
val to_string : t -> string
Encode as a string (not to be used for user-facing messages).
val print : t -> Pp.t
Print internal representation (not to be used for user-facing messages).
val debug_to_string : t -> string
Same as to_string, but outputs extra information related to debug.
to_string
val debug_print : t -> Pp.t
Same as print, but outputs extra information related to debug.
print