aboutsummaryrefslogtreecommitdiffhomepage
path: root/isar/Example-Tokens.thy
diff options
context:
space:
mode:
authorGravatar David Aspinall <da@inf.ed.ac.uk>2008-07-24 09:51:53 +0000
committerGravatar David Aspinall <da@inf.ed.ac.uk>2008-07-24 09:51:53 +0000
commit76d6b0b2b1f039549d308a0d2c478a6b05869af9 (patch)
tree78cc7e13bf290a17e7006a6d4616a8a08e36ce8f /isar/Example-Tokens.thy
parent8f8e9388b582ad6d3ee6e1eea842a8d443d4ce89 (diff)
Merge changes from Version4Branch.
Diffstat (limited to 'isar/Example-Tokens.thy')
-rw-r--r--isar/Example-Tokens.thy34
1 files changed, 34 insertions, 0 deletions
diff --git a/isar/Example-Tokens.thy b/isar/Example-Tokens.thy
new file mode 100644
index 00000000..2eee4f18
--- /dev/null
+++ b/isar/Example-Tokens.thy
@@ -0,0 +1,34 @@
+(*
+ Example proof document for Isabelle/Isar Proof General,
+ using symbols.
+ View and process this document with Unicode Tokens engaged.
+
+ $Id$
+*)
+
+theory "Example-Xsym" imports Main begin
+
+text {* Proper proof text -- \<^bitalic>naive version\<^eitalic>. *}
+
+theorem and_comms: "\<phi> \<and> \<psi> \<longrightarrow> \<psi> \<and> \<phi>"
+proof
+ assume "\<phi> \<and> \<psi>"
+ then show "\<psi> \<and> \<phi>"
+ proof
+ assume \<psi> and \<phi>
+ then show ?thesis ..
+ qed
+qed
+
+text {* \<^bbold>Unstructured\<^ebold> proof script. *}
+
+theorem "\<phi>\<^isub>\<alpha> \<and> \<phi>\<^isub>\<beta> \<longrightarrow> (\<phi>\<^isub>\<beta> ∧ \<phi>\<^isub>\<alpha>)"
+ apply (rule impI)
+ apply (erule conjE)
+ apply (rule conjI)
+ apply assumption
+ apply assumption
+done
+
+end
+