aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/extraction/extraction.mli
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-07-16 12:45:39 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-07-16 12:45:39 +0000
commitf71117475f0ae994c107c7b9e7ea48c9a7a6514f (patch)
tree70be735b5a47ba3a272def311e2b66fea3744993 /contrib/extraction/extraction.mli
parentea41376804c30a583377c0ca45ad8e1b378838df (diff)
Gros Remaniement Extraction:
* extraction.ml + modulaire (cf extract_type) et + proche theorie (cf feu extract_app) * table.ml filtre les Extract Constant vers types ou terms * extract_env.ml refuse maintenant les Extraction constr. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2886 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/extraction/extraction.mli')
-rw-r--r--contrib/extraction/extraction.mli16
1 files changed, 0 insertions, 16 deletions
diff --git a/contrib/extraction/extraction.mli b/contrib/extraction/extraction.mli
index d48fde802..fe57be427 100644
--- a/contrib/extraction/extraction.mli
+++ b/contrib/extraction/extraction.mli
@@ -10,24 +10,9 @@
(*s Extraction from Coq terms to Miniml. *)
-open Names
-open Term
open Miniml
-open Environ
open Nametab
-(*s Result of an extraction. *)
-
-type signature = bool list
-
-type extraction_result =
- | Emltype of ml_type * signature * identifier list
- | Emlterm of ml_ast
-
-(*s Extraction function. *)
-
-val extract_constr : env -> constr -> extraction_result
-
(*s ML declaration corresponding to a Coq reference. *)
val extract_declaration : global_reference -> ml_decl
@@ -41,4 +26,3 @@ val decl_is_logical_ind : global_reference -> bool
val decl_is_singleton : global_reference -> bool
-val extract_type : env -> constr -> constr list -> int list -> ml_type