package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
type global_reference = Names.global_reference =
  1. | VarRef of Names.variable
  2. | ConstRef of Names.Constant.t
  3. | IndRef of Names.inductive
  4. | ConstructRef of Names.constructor
val isVarRef : global_reference -> bool
val isConstRef : global_reference -> bool
val isIndRef : global_reference -> bool
val isConstructRef : global_reference -> bool
val eq_gr : global_reference -> global_reference -> bool
val canonical_gr : global_reference -> global_reference
val destVarRef : global_reference -> Names.variable
val destConstRef : global_reference -> Names.Constant.t
val destIndRef : global_reference -> Names.inductive
val destConstructRef : global_reference -> Names.constructor
val is_global : global_reference -> Constr.constr -> bool
val subst_global_reference : Mod_subst.substitution -> global_reference -> global_reference
val printable_constr_of_global : global_reference -> Constr.constr
val global_of_constr : Constr.constr -> global_reference
val reference_of_constr : Constr.constr -> global_reference
  • deprecated Alias of Globnames.global_of_constr
module RefOrdered : sig ... end
module RefOrdered_env : sig ... end
module Refset : sig ... end
module Refmap : sig ... end
module Refset_env : sig ... end
module Refmap_env : sig ... end
type syndef_name = Names.KerName.t
type extended_global_reference =
  1. | TrueGlobal of global_reference
  2. | SynDef of syndef_name
module ExtRefOrdered : sig ... end
type global_reference_or_constr =
  1. | IsGlobal of global_reference
  2. | IsConstr of Constr.constr
val encode_mind : Names.DirPath.t -> Names.Id.t -> Names.MutInd.t
val pop_global_reference : global_reference -> global_reference
OCaml

Innovation. Community. Security.