diff options
| author | coq | 2002-08-02 17:17:42 +0000 |
|---|---|---|
| committer | coq | 2002-08-02 17:17:42 +0000 |
| commit | 12965209478bd99dfbe57f07d5b525e51b903f22 (patch) | |
| tree | 36a7f5e4802cd321caf02fed0be8349100be09fb /test-suite/modules/fun_objects.v | |
| parent | 8b26fd6ba739d4f49fae99ed764b086022e44b50 (diff) | |
Modules dans COQ\!\!\!\!
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2957 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/modules/fun_objects.v')
| -rw-r--r-- | test-suite/modules/fun_objects.v | 32 |
1 files changed, 32 insertions, 0 deletions
diff --git a/test-suite/modules/fun_objects.v b/test-suite/modules/fun_objects.v new file mode 100644 index 0000000000..b14c3f7935 --- /dev/null +++ b/test-suite/modules/fun_objects.v @@ -0,0 +1,32 @@ +Implicit Arguments On. + +Modtype SIG. + Parameter id:(A:Set)A->A. +EndT SIG. + +Mod M[X:SIG]. + Definition idid := (X.id X.id). + Definition id := (idid X.id). +EndM M. + +Mod N:=M. + +Mod Nat. + Definition T := nat. + Definition x := O. + Definition id := [A:Set][x:A]x. +EndM Nat. + +Mod Z:=(N Nat). + +Check (Z.idid O). + +Mod P[Y:SIG] := N. + +Mod Y:=P Nat Z. + +Check (Y.id O). + + + + |
