aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-10 02:30:55 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-10 02:30:55 +0000
commit53e3a6a6d2d9673f8ba83797b0cdf1ec37f0fd7c (patch)
treeee211bb97ba2f9c80c0bc1bfd059c6ed6ca78067 /contrib
parent1347a59b1198dabbcb6e8a697d896804d533c8d3 (diff)
le pb du <<.v vu comme module>> engendre maintenant une erreur
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4851 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib')
-rw-r--r--contrib/extraction/extract_env.ml1
-rw-r--r--contrib/extraction/table.ml4
-rw-r--r--contrib/extraction/table.mli1
3 files changed, 6 insertions, 0 deletions
diff --git a/contrib/extraction/extract_env.ml b/contrib/extraction/extract_env.ml
index 972c8931c..dd95195ee 100644
--- a/contrib/extraction/extract_env.ml
+++ b/contrib/extraction/extract_env.ml
@@ -183,6 +183,7 @@ let rec extract_msb env v mp all = function
else ms
and extract_meb env v mpo all = function
+ | MEBident (MPfile d) -> error_MPfile_as_mod d (* temporary (I hope) *)
| MEBident mp -> visit_mp v mp; MEident mp
| MEBapply (meb, meb',_) ->
MEapply (extract_meb env v None true meb,
diff --git a/contrib/extraction/table.ml b/contrib/extraction/table.ml
index 96da2259d..8f263015b 100644
--- a/contrib/extraction/table.ml
+++ b/contrib/extraction/table.ml
@@ -192,6 +192,10 @@ let error_unqualified_name s1 s2 =
"in ML from another name sharing the same basename.\n" ^
"Please do some renaming.\n"))
+let error_MPfile_as_mod d =
+ err (str ("The whole file "^(string_of_dirpath d)^".v is used somewhere as a module.\n"^
+ "Extraction cannot currently deal with this situation.\n"))
+
(*S The Extraction auxiliary commands *)
(*s Extraction AutoInline *)
diff --git a/contrib/extraction/table.mli b/contrib/extraction/table.mli
index 1e8371d1e..6e413b626 100644
--- a/contrib/extraction/table.mli
+++ b/contrib/extraction/table.mli
@@ -28,6 +28,7 @@ val error_toplevel : unit -> 'a
val error_scheme : unit -> 'a
val error_not_visible : global_reference -> 'a
val error_unqualified_name : string -> string -> 'a
+val error_MPfile_as_mod : dir_path -> 'a
val check_inside_module : unit -> unit
val check_inside_section : unit -> unit