aboutsummaryrefslogtreecommitdiff
path: root/coq/example.v
diff options
context:
space:
mode:
authorPierre Courtieu2003-01-29 18:56:05 +0000
committerPierre Courtieu2003-01-29 18:56:05 +0000
commitd4b3bb61d84cb2cd831a43b65dc55ef25fa8abaa (patch)
tree2747f268bfc5d439931f41bd845e3ce9e236ed88 /coq/example.v
parenta87f482d11b56fd8d3bbe148e174c4010e327794 (diff)
Added a file for testing modules of coq (new version 7.4). Plus some
modification to better backtrack modules.
Diffstat (limited to 'coq/example.v')
-rw-r--r--coq/example.v6
1 files changed, 5 insertions, 1 deletions
diff --git a/coq/example.v b/coq/example.v
index 5d55a2ae..6f92e279 100644
--- a/coq/example.v
+++ b/coq/example.v
@@ -9,7 +9,7 @@
$Id$
*)
-Section sect.
+Module sect.
Goal (A,B:Prop)(A /\ B) -> (B /\ A).
Intros A B H.
@@ -32,5 +32,9 @@ End mod.
Module Type newmod.
Definition type1:=Set.
+
+Goal (n:nat)n=n.
+Auto.
+Save toto.
End newmod.