aboutsummaryrefslogtreecommitdiffhomepage
path: root/isar/Example.thy
diff options
context:
space:
mode:
authorGravatar David Aspinall <da@inf.ed.ac.uk>2000-06-01 13:41:31 +0000
committerGravatar David Aspinall <da@inf.ed.ac.uk>2000-06-01 13:41:31 +0000
commitbfd4724e70dd6e03fe8f391b7736ce67b15b3616 (patch)
treeb4262a30004d5053c0ba339edd6471f23a91de7e /isar/Example.thy
parent4dde556b466b81b864e65ccaa0401e121dc27f1a (diff)
Removed now spurious semicolons, 8-).
Diffstat (limited to 'isar/Example.thy')
-rw-r--r--isar/Example.thy25
1 files changed, 12 insertions, 13 deletions
diff --git a/isar/Example.thy b/isar/Example.thy
index f6500e6d..7b4fdcac 100644
--- a/isar/Example.thy
+++ b/isar/Example.thy
@@ -8,17 +8,16 @@
you may get the theory mode of ordinary Isabelle Proof General
*)
+theory Example = Main:
-theory Example = Main:;
-
-theorem and_comms: "A & B --> B & A";
-proof;
- assume "A & B";
- thus "B & A";
- proof;
- assume A B;
- show ?thesis; ..;
- qed;
-qed;
-
-end;
+theorem and_comms: "A & B --> B & A"
+proof
+ assume "A & B"
+ thus "B & A"
+ proof
+ assume A B
+ show ?thesis
+ ..
+ qed
+qed
+end