From b03ab4806e33a5f0a808d6325b87ab95189cd460 Mon Sep 17 00:00:00 2001 From: David Aspinall Date: Thu, 22 Apr 2004 10:21:05 +0000 Subject: Update to Coq 8.0 syntax --- coq/ex-module.v | 6 +++--- 1 file changed, 3 insertions(+), 3 deletions(-) (limited to 'coq/ex-module.v') 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. -- cgit v1.2.3