aboutsummaryrefslogtreecommitdiff
path: root/test-suite/output/PrintModule.out
blob: 7c7600b786633d26a7a60141962639e403f2a14d (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
Module N : S with Definition T := nat := M

Module N : S with Definition T := M

Module N : S with Module T := K := M

Module N : S with Module T := M

Module Type Func = Funsig (T0:Test) Sig Parameter x : T0.t. End
Module
A
:= Struct
     Variant I : Set :=  C : nat -> I.
     Record R : Set := Build_R { n : nat }.
     Definition n : R -> nat.
   End