aboutsummaryrefslogtreecommitdiffhomepage
path: root/isar/Example.thy
diff options
context:
space:
mode:
authorGravatar Makarius Wenzel <makarius@sketis.net>1999-05-27 19:27:27 +0000
committerGravatar Makarius Wenzel <makarius@sketis.net>1999-05-27 19:27:27 +0000
commitde6ec194f89ccf50b55109957cc6eae9bbec5307 (patch)
tree800146d8b21f37f9bcb8f51e724728c18713b005 /isar/Example.thy
parentbb675ae202e887b2a47d57d0aecbec1bfa8794ba (diff)
be chatty;
Diffstat (limited to 'isar/Example.thy')
-rw-r--r--isar/Example.thy9
1 files changed, 9 insertions, 0 deletions
diff --git a/isar/Example.thy b/isar/Example.thy
index 8dc4b04a..f9807888 100644
--- a/isar/Example.thy
+++ b/isar/Example.thy
@@ -1,6 +1,10 @@
theory Example = Main:;
+text {*
+ Just a few tiny examples to get an idea of how Isabelle/Isar proof documents
+ may look like.
+ *}
lemma I: "A --> A";
proof;
@@ -17,6 +21,11 @@ proof;
qed;
qed;
+text {*
+ This one is a good test for ProofGeneral to cope with block-structured
+ proof texts. Have fun with automatic indentation!
+ *};
+
lemma S: "(A --> B --> C) --> (A --> B) --> A --> C";
proof;
assume "A --> B --> C";