aboutsummaryrefslogtreecommitdiffhomepage
path: root/isar/Example.thy
diff options
context:
space:
mode:
authorGravatar David Aspinall <da@inf.ed.ac.uk>2009-09-15 07:48:10 +0000
committerGravatar David Aspinall <da@inf.ed.ac.uk>2009-09-15 07:48:10 +0000
commit93aff45f52f9bf14f64e5b42ef16aa24d15bd79a (patch)
treedcfba599fc18a08596c47ac7ad8845311771b329 /isar/Example.thy
parent682b4c17840aaa694cf3c7684bb5b06bcb4108c2 (diff)
Revert accidental commit
Diffstat (limited to 'isar/Example.thy')
-rw-r--r--isar/Example.thy9
1 files changed, 3 insertions, 6 deletions
diff --git a/isar/Example.thy b/isar/Example.thy
index b0640146..720e5480 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 \<and> B \<longrightarrow> B \<and> A"
+theorem and_comms: "A & B --> B & A"
proof
- assume "A \<and> B"
- then show "B \<and> A"
+ assume "A & B"
+ then show "B & A"
proof
assume B and A
then show ?thesis ..
@@ -22,9 +22,6 @@ qed
text {* Unstructured proof script. *}
theorem "A & B --> B & A"
-by and_comms
-
-
apply (rule impI)
apply (erule conjE)
apply (rule conjI)