aboutsummaryrefslogtreecommitdiffhomepage
path: root/library/declare.mli
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-11-05 16:48:30 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-11-05 16:48:30 +0000
commitb91f60aab99980b604dc379b4ca62f152315c841 (patch)
treecd1948fc5156988dd74d94ef4abb3e4ac77e3de8 /library/declare.mli
parent2ff72589e5c90a25b315922b5ba2d7c11698adef (diff)
GROS COMMIT:
- reduction du noyau (variables existentielles, fonctions auxiliaires pour inventer des noms, etc. deplacees hors de kernel/) - changement de noms de constructeurs des constr (suppression de "Is" et "Mut") git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2158 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'library/declare.mli')
-rw-r--r--library/declare.mli24
1 files changed, 6 insertions, 18 deletions
diff --git a/library/declare.mli b/library/declare.mli
index be5678f7f..c57dd2079 100644
--- a/library/declare.mli
+++ b/library/declare.mli
@@ -13,8 +13,10 @@ open Names
open Term
open Sign
open Declarations
-open Inductive
+open Indtypes
+open Safe_typing
open Library
+open Nametab
(*i*)
(* This module provides the official functions to declare new variables,
@@ -33,9 +35,9 @@ type section_variable_entry =
| SectionLocalDef of constr
| SectionLocalAssum of constr
-type variable_declaration = section_variable_entry * strength
+type variable_declaration = dir_path * section_variable_entry * strength
-val declare_variable : identifier -> variable_declaration -> variable
+val declare_variable : variable -> variable_declaration -> section_path
type constant_declaration_type =
| ConstantEntry of constant_entry
@@ -57,10 +59,6 @@ val declare_parameter : identifier -> constr -> constant
the whole block *)
val declare_mind : mutual_inductive_entry -> mutual_inductive
-(* [declare_eliminations sp] declares elimination schemes associated
- to the mutual inductive block refered by [sp] *)
-val declare_eliminations : mutual_inductive -> unit
-
val out_inductive : Libobject.obj -> mutual_inductive_entry
val make_strength_0 : unit -> strength
@@ -78,13 +76,12 @@ val get_variable : variable -> named_declaration * strength
val get_variable_with_constraints :
variable -> named_declaration * Univ.constraints * strength
val variable_strength : variable -> strength
-val find_section_variable : identifier -> variable
+val find_section_variable : variable -> section_path
val last_section_hyps : dir_path -> identifier list
(*s Global references *)
val context_of_global_reference : global_reference -> section_context
-val extract_instance : global_reference -> constr array -> constr array
(* Turn a global reference into a construction *)
val constr_of_reference : global_reference -> constr
@@ -108,12 +105,3 @@ val global_reference : identifier -> constr
val construct_reference : Environ.env -> identifier -> constr
val is_global : identifier -> bool
-
-val path_of_inductive_path : inductive -> mutual_inductive
-val path_of_constructor_path : constructor -> mutual_inductive
-
-(* Look up function for the default elimination constant *)
-val elimination_suffix : sorts_family -> string
-val make_elimination_ident :
- inductive_ident:identifier -> sorts_family -> identifier
-val lookup_eliminator : Environ.env -> inductive -> sorts_family -> constr