blob: 45cf9f12421d983ab322dd45287e28ce251f17b6 (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
|
Module M.
Definition T := nat.
Definition x : T := 0.
End M.
Module Type SIG.
Module M := Top.M.
Module Type SIG.
Parameter T : Set.
End SIG.
Declare Module N: SIG.
End SIG.
Module Z.
Module M := Top.M.
Module Type SIG.
Parameter T : Set.
End SIG.
Module N := M.
End Z.
Module A : SIG := Z.
|