From 6d961ac24305f26e896b602bdabe0e9c3c7cbf05 Mon Sep 17 00:00:00 2001 From: letouzey Date: Tue, 29 May 2012 11:09:15 +0000 Subject: global_reference migrated from Libnames to new Globnames, less deps in grammar.cma git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15384 85f007b7-540e-0410-9357-904b9bb8a0f7 --- library/libnames.mli | 77 ---------------------------------------------------- 1 file changed, 77 deletions(-) (limited to 'library/libnames.mli') diff --git a/library/libnames.mli b/library/libnames.mli index d3eed0364..0fe687343 100644 --- a/library/libnames.mli +++ b/library/libnames.mli @@ -10,69 +10,6 @@ open Pp open Errors open Util open Names -open Term -open Mod_subst - -(** {6 Global reference is a kernel side type for all references together } *) -type global_reference = - | VarRef of variable - | ConstRef of constant - | IndRef of inductive - | ConstructRef of 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 -> variable -val destConstRef : global_reference -> constant -val destIndRef : global_reference -> inductive -val destConstructRef : global_reference -> constructor - - -val subst_constructor : substitution -> constructor -> constructor * constr -val subst_global : substitution -> global_reference -> global_reference * constr - -(** Turn a global reference into a construction *) -val constr_of_global : global_reference -> constr - -(** Turn a construction denoting a global reference into a global reference; - raise [Not_found] if not a global reference *) -val global_of_constr : constr -> global_reference - -(** Obsolete synonyms for constr_of_global and global_of_constr *) -val constr_of_reference : global_reference -> constr -val reference_of_constr : constr -> global_reference - -module RefOrdered : sig - type t = global_reference - val compare : global_reference -> global_reference -> int -end - -module RefOrdered_env : sig - type t = global_reference - val compare : global_reference -> global_reference -> int -end - -module Refset : Set.S with type elt = global_reference -module Refmap : Map.S with type key = global_reference - -(** {6 Extended global references } *) - -type syndef_name = kernel_name - -type extended_global_reference = - | TrueGlobal of global_reference - | SynDef of syndef_name - -module ExtRefOrdered : sig - type t = extended_global_reference - val compare : t -> t -> int -end (** {6 Dirpaths } *) val pr_dirpath : dir_path -> Pp.std_ppcmds @@ -121,14 +58,6 @@ module Spmap : Map.S with type key = full_path val restrict_path : int -> full_path -> full_path -(** {6 Temporary function to brutally form kernel names from section paths } *) - -val encode_mind : dir_path -> identifier -> mutual_inductive -val decode_mind : mutual_inductive -> dir_path * identifier -val encode_con : dir_path -> identifier -> constant -val decode_con : constant -> dir_path * identifier - - (** {6 ... } *) (** A [qualid] is a partially qualified ident; it includes fully qualified names (= absolute names) and all intermediate partial @@ -184,12 +113,6 @@ val string_of_reference : reference -> string val pr_reference : reference -> std_ppcmds val loc_of_reference : reference -> loc -(** {6 Popping one level of section in global names } *) - -val pop_con : constant -> constant -val pop_kn : mutual_inductive-> mutual_inductive -val pop_global_reference : global_reference -> global_reference - (** Deprecated synonyms *) val make_short_qualid : identifier -> qualid (** = qualid_of_ident *) -- cgit v1.2.3