aboutsummaryrefslogtreecommitdiffhomepage
path: root/etc/coq/nested.v
diff options
context:
space:
mode:
authorGravatar David Aspinall <da@inf.ed.ac.uk>2002-06-11 10:54:52 +0000
committerGravatar David Aspinall <da@inf.ed.ac.uk>2002-06-11 10:54:52 +0000
commitef1b6fd069272733ee9f06ba03215ef7702a1aa8 (patch)
tree04833557014d2d69a7df43cb7d01dd82fd98c640 /etc/coq/nested.v
parentf89b20c5d5fb332581d67f4d689a22e8ef95f02f (diff)
New files.
Diffstat (limited to 'etc/coq/nested.v')
-rw-r--r--etc/coq/nested.v19
1 files changed, 19 insertions, 0 deletions
diff --git a/etc/coq/nested.v b/etc/coq/nested.v
new file mode 100644
index 00000000..db7608ea
--- /dev/null
+++ b/etc/coq/nested.v
@@ -0,0 +1,19 @@
+(*
+ Example nested proof script for testing support of nested proofs.
+*)
+
+Goal (A,B:Prop)(A /\ B) -> (B /\ A).
+ Intros A B H.
+ Induction H.
+ Apply conj.
+ Lemma foo: (A,B:Prop)(A /\ B) -> (B /\ A).
+ Intros A B H.
+ Induction H.
+ Apply conj.
+ Assumption.
+ Assumption.
+ Save.
+ Assumption.
+ Assumption.
+Save and_comms.
+