blob: c09a74324138c8af5954c04099d49f98652074bc (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
|
Module M.
Module Type SIG.
Parameter T:Set.
Parameter x:T.
End SIG.
Module N:SIG.
Definition T:=nat.
Definition x:=O.
End N.
End M.
Module N:=M.
Module Type SPRYT.
Module N.
Definition T:=M.N.T.
Parameter x:T.
End N.
End SPRYT.
Module K:SPRYT:=N.
Module K':SPRYT:=M.
Module Type SIG.
Definition T:Set:=M.N.T.
Parameter x:T.
End SIG.
Module J:SIG:=M.N.
|