summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/shouldsucceed/2608.v
diff options
context:
space:
mode:
authorGravatar Stephane Glondu <steph@glondu.net>2011-12-25 13:19:42 +0100
committerGravatar Stephane Glondu <steph@glondu.net>2011-12-25 13:19:42 +0100
commit300293c119981054c95182a90c829058530a6b6f (patch)
treed7303613741c5796b58ced7db24ec7203327dbb2 /test-suite/bugs/closed/shouldsucceed/2608.v
parent9d27ae09786866b6e3d7b79d1fa7667e5e2aa309 (diff)
Imported Upstream version 8.3.pl3upstream/8.3.pl3
Diffstat (limited to 'test-suite/bugs/closed/shouldsucceed/2608.v')
-rw-r--r--test-suite/bugs/closed/shouldsucceed/2608.v34
1 files changed, 34 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/shouldsucceed/2608.v b/test-suite/bugs/closed/shouldsucceed/2608.v
new file mode 100644
index 00000000..a4c95ff9
--- /dev/null
+++ b/test-suite/bugs/closed/shouldsucceed/2608.v
@@ -0,0 +1,34 @@
+
+Module Type T.
+ Parameter Inline t : Type.
+End T.
+
+Module M.
+ Definition t := nat.
+End M.
+
+Module Make (X:T).
+ Include X.
+
+ (* here t is : (Top.Make.t,Top.X.t) *)
+
+ (* in libobject HEAD : EvalConstRef (Top.X.t,Top.X.t)
+ which is substituted by : {Top.X |-> Top.Make [, Top.Make.t=>Top.X.t]}
+ which gives : EvalConstRef (Top.Make.t,Top.X.t) *)
+
+End Make.
+
+Module P := Make M.
+
+ (* resolver returned by add_module : Top.P.t=>inline *)
+ (* then constant_of_delta_kn P.t produces (Top.P.t,Top.P.t) *)
+
+ (* in libobject HEAD : EvalConstRef (Top.Make.t,Top.X.t)
+ given to subst = {<X#1> |-> Top.M [, Top.M.t=>inline]}
+ which used to give : EvalConstRef (Top.Make.t,Top.M.t)
+ given to subst = {Top.Make |-> Top.P [, Top.P.t=>inline]}
+ which used to give : EvalConstRef (Top.P.t,Top.M.t) *)
+
+Definition u := P.t.
+ (* was raising Not_found since Heads.head_map knows of (Top.P.t,Top.M.t)
+ and not of (Top.P.t,Top.P.t) *)