aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/extraction/table.mli
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-12-09 02:14:55 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-12-09 02:14:55 +0000
commit3b05f397df3af10604d0abaa82fc55ff4ef189eb (patch)
treec97894871b73a7da6179c1f04b3d29954e0867db /contrib/extraction/table.mli
parent0c3b7fd6677de61e435bbdbd89bcf3758396ef41 (diff)
chamboulement du codage des indcutifs extraits; deplacements des tables; ...
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3388 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/extraction/table.mli')
-rw-r--r--contrib/extraction/table.mli44
1 files changed, 23 insertions, 21 deletions
diff --git a/contrib/extraction/table.mli b/contrib/extraction/table.mli
index 3ffb74ac4..e6495add6 100644
--- a/contrib/extraction/table.mli
+++ b/contrib/extraction/table.mli
@@ -10,16 +10,18 @@
open Names
open Libnames
+open Miniml
(*s Warning and Error messages. *)
+val error_axiom_scheme : global_reference -> 'a
+val error_axiom : global_reference -> 'a
+val warning_axiom : global_reference -> unit
val error_section : unit -> 'a
-
-val error_axiom_scheme : kernel_name -> 'a
-
-val error_axiom : kernel_name -> 'a
-
-val warning_axiom : kernel_name -> unit
+val error_constant : global_reference -> 'a
+val error_type_scheme : global_reference -> 'a
+val error_inductive : global_reference -> 'a
+val error_nb_cons : unit -> 'a
(*s AutoInline parameter *)
@@ -32,46 +34,46 @@ val optim : unit -> bool
(*s Target language. *)
type lang = Ocaml | Haskell | Scheme | Toplevel
-
val lang : unit -> lang
(*s Table for custom inlining *)
val to_inline : global_reference -> bool
-
val to_keep : global_reference -> bool
(*s Table for direct ML extractions. *)
val is_ml_extraction : global_reference -> bool
-
val find_ml_extraction : global_reference -> string
-
val ml_extractions : unit -> Refset.t
-
val ml_type_extractions : unit -> (global_reference * string) list
-
val ml_term_extractions : unit -> (global_reference * string) list
(*s Extraction commands. *)
val extraction_language : lang -> unit
-
val extraction_inline : bool -> reference list -> unit
-
val print_extraction_inline : unit -> unit
-
val reset_extraction_inline : unit -> unit
-
val extract_constant_inline : bool -> reference -> string -> unit
-
val extract_inductive : reference -> string * string list -> unit
-(*s some tables. *)
+(*s Some table-related operations *)
+
+val add_term : kernel_name -> ml_decl -> unit
+val lookup_term : kernel_name -> ml_decl
-val add_record : inductive -> global_reference list -> unit
-val find_proj : inductive -> global_reference list
-val is_proj : global_reference -> bool
+val add_type : kernel_name -> ml_schema -> unit
+val lookup_type : kernel_name -> ml_schema
+
+val add_ind : kernel_name -> ml_ind -> unit
+val lookup_ind : kernel_name -> ml_ind
val add_recursors : kernel_name -> unit
val is_recursor : global_reference -> bool
+
+val add_record : kernel_name -> global_reference list -> unit
+val find_projections : kernel_name -> global_reference list
+val is_projection : global_reference -> bool
+
+