aboutsummaryrefslogtreecommitdiffhomepage
path: root/isar/Example.thy
diff options
context:
space:
mode:
authorGravatar Makarius Wenzel <makarius@sketis.net>2001-09-04 19:19:57 +0000
committerGravatar Makarius Wenzel <makarius@sketis.net>2001-09-04 19:19:57 +0000
commit876bf804fcd7ed07c6b6cd8af5f5ac0bf348eea1 (patch)
tree6852ad124536de3f7bc5a2b29e4dcea0b5585aee /isar/Example.thy
parentb1e40009c84d0deffa99492c63b2fdb93196d5ce (diff)
tuned proof text;
added script version;
Diffstat (limited to 'isar/Example.thy')
-rw-r--r--isar/Example.thy18
1 files changed, 15 insertions, 3 deletions
diff --git a/isar/Example.thy b/isar/Example.thy
index 22c0a4e1..179b5b83 100644
--- a/isar/Example.thy
+++ b/isar/Example.thy
@@ -11,15 +11,27 @@
theory Example = Main:
+text {* Proper proof text. *}
+
theorem and_comms: "A & B --> B & A"
proof
assume "A & B"
thus "B & A"
proof
- assume A B
- show ?thesis
- ..
+ assume B and A
+ thus ?thesis ..
qed
qed
+
+text {* Proof script. *}
+
+theorem "A & B --> B & A"
+ apply (rule impI)
+ apply (erule conjE)
+ apply (rule conjI)
+ apply assumption
+ apply assumption
+ done
+
end