aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex-module.v
diff options
context:
space:
mode:
authorGravatar Pierre Courtieu <courtieu@lri.fr>2007-04-16 14:28:26 +0000
committerGravatar Pierre Courtieu <courtieu@lri.fr>2007-04-16 14:28:26 +0000
commit9093e9c24213318a27888363b72659d05ce1ff6c (patch)
treecd707c2d04600ef1a6701df14ef200c091862874 /coq/ex-module.v
parentd6460395d8004d1774241bca5e52bb168f62a144 (diff)
Small fixes from Stefan Monnier.
Diffstat (limited to 'coq/ex-module.v')
-rw-r--r--coq/ex-module.v20
1 files changed, 12 insertions, 8 deletions
diff --git a/coq/ex-module.v b/coq/ex-module.v
index 413a4966..e6e3511f 100644
--- a/coq/ex-module.v
+++ b/coq/ex-module.v
@@ -1,4 +1,4 @@
-
+(* *)
Module Type O1.
Parameter A:Set.
Parameter B:Set.
@@ -24,18 +24,22 @@ End R4.
Module M.
+
Module Type SIG.
Parameter T:Set.
Parameter x:T.
End SIG.
+
Module Type SIG'.
Parameter T:Set.
Parameter x:T.
End SIG'.
+
Lemma toto : O=O.
Definition t:=nat.
trivial.
Save.
+
Module N:SIG.
Definition T:=nat.
Definition x:=O.
@@ -71,16 +75,16 @@ Module Type N'.
Declare Module K:N.SIG.
End M'.
(* Declare Module N''. *)
- Definition T:=nat.
- Definition x:=O.
+ Definition T:=nat.
+ Definition x:=O.
(* End N''. *)
Declare Module N':M.SIG. (* no interactive def started *)
Declare Module N''' :M.SIG. (* no interactive def started *)
End N'.
-
-
+
+
Lemma titi : O=O.
trivial.
Module Type K:=N'.
@@ -88,9 +92,9 @@ Lemma titi : O=O.
Save.
(* Here is a bug of Coq: *)
-
+
Lemma bar:O=O.
Module Type L. (* This should not be allowed by Coq, since the End L. below fails *)
- End L. (* fails --> if we go back to Module Type: unsync *)
- Module I.
+End L. (* fails --> if we go back to Module Type: unsync *)
+Module I.
End I.