aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex-module.v
diff options
context:
space:
mode:
authorGravatar Pierre Courtieu <courtieu@lri.fr>2006-04-26 22:31:52 +0000
committerGravatar Pierre Courtieu <courtieu@lri.fr>2006-04-26 22:31:52 +0000
commit8ba99b2013e0f62c9117fc79364630ff1fbec585 (patch)
tree1ecc9083150779a527fab764508ac9dab7d78096 /coq/ex-module.v
parentfc774de804417a399094f61de1880e75b556c851 (diff)
Changed the type of proof-goal-command-p. It takes now a span, which
allows using a span attribute to detect goal commands. I think I modified all modes accordingly.
Diffstat (limited to 'coq/ex-module.v')
-rw-r--r--coq/ex-module.v14
1 files changed, 7 insertions, 7 deletions
diff --git a/coq/ex-module.v b/coq/ex-module.v
index 5b9d638a..413a4966 100644
--- a/coq/ex-module.v
+++ b/coq/ex-module.v
@@ -28,6 +28,10 @@ Module M.
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.
@@ -66,16 +70,13 @@ Module Type N'.
Module Type M'.
Declare Module K:N.SIG.
End M'.
- Declare Module N''.
+(* Declare Module N''. *)
Definition T:=nat.
Definition x:=O.
- End N''.
+(* End N''. *)
Declare Module N':M.SIG. (* no interactive def started *)
- Declare Module N''':= N'. (* no interactive def started *)
- Declare Module N''''. (* interactive def started *)
- Parameter foo:nat.
- End N''''. (* interactive def ended *)
+ Declare Module N''' :M.SIG. (* no interactive def started *)
End N'.
@@ -90,7 +91,6 @@ Save.
Lemma bar:O=O.
Module Type L. (* This should not be allowed by Coq, since the End L. below fails *)
- Axiom foo: O=O.
End L. (* fails --> if we go back to Module Type: unsync *)
Module I.
End I.