aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/PrintModule.v
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2015-07-27 13:58:05 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2015-07-27 13:59:30 +0200
commitcb145fa37d463210832c437f013231c9f028e1aa (patch)
tree85214302c2c0e33b587f2e4eb87a3ba2b0a4a7c7 /test-suite/output/PrintModule.v
parentcf193df65c53813054239463f6496526533e9bab (diff)
Output test for bug #2169.
Diffstat (limited to 'test-suite/output/PrintModule.v')
-rw-r--r--test-suite/output/PrintModule.v34
1 files changed, 34 insertions, 0 deletions
diff --git a/test-suite/output/PrintModule.v b/test-suite/output/PrintModule.v
new file mode 100644
index 000000000..999d9a986
--- /dev/null
+++ b/test-suite/output/PrintModule.v
@@ -0,0 +1,34 @@
+Module FOO.
+
+Module M.
+ Definition T := nat.
+End M.
+
+Module Type S.
+ Parameter T : Set.
+End S.
+
+Module N : S with Definition T := nat := M.
+
+Print Module N.
+
+End FOO.
+
+Module BAR.
+
+Module K. End K.
+Module Type KS. End KS.
+
+Module M.
+ Module T := K.
+End M.
+
+Module Type S.
+ Declare Module T : KS.
+End S.
+
+Module N : S with Module T := K := M.
+
+Print Module N.
+
+End BAR.