aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel
diff options
context:
space:
mode:
authorGravatar coq <coq@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-01-22 10:04:13 +0000
committerGravatar coq <coq@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-01-22 10:04:13 +0000
commit314333e2ce7c06293ab6e5292b2927afb75b6a6f (patch)
tree0af2af425e99e771a9279616850f660a97a1f60b /kernel
parente4c997965f822488376fde2bb34285d3ec943a20 (diff)
Bug 'with Module' corrige
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3573 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel')
-rw-r--r--kernel/mod_typing.ml10
-rw-r--r--kernel/modops.ml3
-rw-r--r--kernel/modops.mli2
3 files changed, 14 insertions, 1 deletions
diff --git a/kernel/mod_typing.ml b/kernel/mod_typing.ml
index 7417b4261..8fee8481d 100644
--- a/kernel/mod_typing.ml
+++ b/kernel/mod_typing.ml
@@ -108,7 +108,15 @@ and merge_with env mtb with_decl =
| _ -> error_not_a_module (string_of_label l)
in
let mtb = type_modpath env' mp in
- (* here, we should assert that there is no msid in mtb *)
+ (* here, using assertions in substitutions,
+ we check that there is no msid bound in mtb *)
+ begin
+ try
+ let _ = subst_modtype (map_msid msid (MPself msid)) mtb in
+ ()
+ with
+ Assert_failure _ -> error_circular_with_module id
+ end;
let cst = check_subtypes env' mtb old.msb_modtype in
let equiv =
match old.msb_equiv with
diff --git a/kernel/modops.ml b/kernel/modops.ml
index ec25459a9..c194a6c71 100644
--- a/kernel/modops.ml
+++ b/kernel/modops.ml
@@ -74,6 +74,9 @@ let error_local_context lo =
error ("The local context of the component "^
(string_of_label l)^" is not empty")
+let error_circular_with_module l =
+ error ("The construction \"with Module "^(string_of_id l)^":=...\" is about to create\na circular module type. Their resolution is not implemented yet.\nIf you really need that feature, please report.")
+
let rec scrape_modtype env = function
| MTBident kn -> scrape_modtype env (lookup_modtype kn env)
| mtb -> mtb
diff --git a/kernel/modops.mli b/kernel/modops.mli
index aaff57223..1391380b1 100644
--- a/kernel/modops.mli
+++ b/kernel/modops.mli
@@ -92,3 +92,5 @@ val error_not_a_constant : label -> 'a
val error_with_incorrect : label -> 'a
val error_local_context : label option -> 'a
+
+val error_circular_with_module : identifier -> 'a