blob: cf5e9b090b5e173c6d5a9e32655cdafbf01e33b1 (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
|
Module Type FOO.
Parameters P Q : Type -> Type.
End FOO.
Module Type BAR.
Declare Module Export foo : FOO.
Parameter f : forall A, P A -> Q A -> A.
End BAR.
Module Type BAZ.
Declare Module Export foo : FOO.
Parameter g : forall A, P A -> Q A -> A.
End BAZ.
Module BAR_FROM_BAZ (baz : BAZ) : BAR.
Import baz.
Module foo <: FOO := foo.
Definition f : forall A, P A -> Q A -> A := g.
End BAR_FROM_BAZ.
|