aboutsummaryrefslogtreecommitdiffhomepage
path: root/isar/Example.thy
diff options
context:
space:
mode:
authorGravatar David Aspinall <da@inf.ed.ac.uk>2009-09-15 07:47:15 +0000
committerGravatar David Aspinall <da@inf.ed.ac.uk>2009-09-15 07:47:15 +0000
commit682b4c17840aaa694cf3c7684bb5b06bcb4108c2 (patch)
tree4eced173d60c3a2c2d81d7c2850364a2d8d06332 /isar/Example.thy
parentb8bdbab2356aa0e68164143d3f78c73ad12197c7 (diff)
Fix compile errors
Diffstat (limited to 'isar/Example.thy')
-rw-r--r--isar/Example.thy9
1 files changed, 6 insertions, 3 deletions
diff --git a/isar/Example.thy b/isar/Example.thy
index 720e5480..b0640146 100644
--- a/isar/Example.thy
+++ b/isar/Example.thy
@@ -9,10 +9,10 @@ theory Example imports Main begin
text {* Proper proof text -- \textit{naive version}. *}
-theorem and_comms: "A & B --> B & A"
+theorem and_comms: "A \<and> B \<longrightarrow> B \<and> A"
proof
- assume "A & B"
- then show "B & A"
+ assume "A \<and> B"
+ then show "B \<and> A"
proof
assume B and A
then show ?thesis ..
@@ -22,6 +22,9 @@ qed
text {* Unstructured proof script. *}
theorem "A & B --> B & A"
+by and_comms
+
+
apply (rule impI)
apply (erule conjE)
apply (rule conjI)