aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/extraction/extraction.mli
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-02-20 15:13:24 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-02-20 15:13:24 +0000
commit3cc15f0b98a8a049f6d2190084dbcbade8e2dd63 (patch)
tree8d7c0158a72c4fdc358c0e172d6ba4d2d42105a3 /contrib/extraction/extraction.mli
parentaa099698be3bfea741bdd8698da52e81ec6cd068 (diff)
mise en place fichiers extraction
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1397 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/extraction/extraction.mli')
-rw-r--r--contrib/extraction/extraction.mli27
1 files changed, 26 insertions, 1 deletions
diff --git a/contrib/extraction/extraction.mli b/contrib/extraction/extraction.mli
index 71c9c9be2..485290b03 100644
--- a/contrib/extraction/extraction.mli
+++ b/contrib/extraction/extraction.mli
@@ -2,7 +2,32 @@
(*i $Id$ i*)
open Names
+open Term
open Miniml
-val extract : section_path list -> ml_decl list
+(*s Renaming issues. *)
+
+val get_global_name : identifier -> identifier
+
+type renaming_function = identifier list -> name -> identifier
+
+module type Renaming = sig
+ val rename_type_parameter : renaming_function
+ val rename_type : renaming_function
+ val rename_term : renaming_function
+ val rename_global_type : renaming_function
+ val rename_global_constructor : renaming_function
+ val rename_global_term : renaming_function
+end
+
+(*s The extraction functor. It returns a single function [extract]
+ translating a piece of CIC environment into a list of ML declarations.
+ The boolean indicates whether cofix are allowed or not. *)
+
+module type Translation = sig
+ val extract : bool -> global_reference list -> ml_decl list
+end
+
+module Make : functor (R : Renaming) -> Translation
+