aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex-module.v
diff options
context:
space:
mode:
authorGravatar David Aspinall <da@inf.ed.ac.uk>2004-04-22 10:21:05 +0000
committerGravatar David Aspinall <da@inf.ed.ac.uk>2004-04-22 10:21:05 +0000
commitb03ab4806e33a5f0a808d6325b87ab95189cd460 (patch)
tree46c2d62dca3d3db5cc796a3e0a82dae79e6f882e /coq/ex-module.v
parent48c7ab576a42556e1891a3ca15225378e49cde48 (diff)
Update to Coq 8.0 syntax
Diffstat (limited to 'coq/ex-module.v')
-rw-r--r--coq/ex-module.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/coq/ex-module.v b/coq/ex-module.v
index af2e4a08..240d0ad1 100644
--- a/coq/ex-module.v
+++ b/coq/ex-module.v
@@ -30,7 +30,7 @@ Module M.
End SIG.
Lemma toto : O=O.
Definition t:=nat.
- Trivial.
+ trivial.
Save.
Module N:SIG.
Definition T:=nat.
@@ -44,7 +44,7 @@ Print t.
Definition t:O=O.
- Trivial.
+ trivial.
Save.
@@ -81,7 +81,7 @@ Module Type N'.
Lemma titi : O=O.
- Trivial.
+ trivial.
Module Type K:=N'.
Module N''':=M.
Save.