aboutsummaryrefslogtreecommitdiffhomepage
path: root/library/declaremods.ml
diff options
context:
space:
mode:
authorGravatar soubiran <soubiran@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-02-10 11:36:01 +0000
committerGravatar soubiran <soubiran@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-02-10 11:36:01 +0000
commitb92c1cd9df6defe7529d79a083b12bf7f5925f2b (patch)
treea88d8c4263fc7ed00443d8414c57645a3f97b465 /library/declaremods.ml
parentb09d87a1cdaa21037b0b1a1b81750c473c22c42d (diff)
Correction bug coqdev Hermann lehener.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11899 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'library/declaremods.ml')
-rw-r--r--library/declaremods.ml1
1 files changed, 1 insertions, 0 deletions
diff --git a/library/declaremods.ml b/library/declaremods.ml
index 16f9c9491..7923f566b 100644
--- a/library/declaremods.ml
+++ b/library/declaremods.ml
@@ -629,6 +629,7 @@ let rec get_modtype_substobjs env = function
| MSEwith (mty, With_Definition _) -> get_modtype_substobjs env mty
| MSEwith (mty, With_Module (idl,mp)) ->
let substobjs = get_modtype_substobjs env mty in
+ let mp = Environ.scrape_alias mp env in
let modobjs = MPmap.find mp !modtab_substobjs in
replace_module_object idl substobjs modobjs mp
| MSEapply (mexpr, MSEident mp) ->