(* Example proof document for Isabelle/Isar Proof General, using symbols. View and process this document with Unicode Tokens engaged. For a more exhaustive test of token display, visit the test file etc/isar/TokensAcid.thy. Check the FAQ for more advice. $Id$ *) theory "Example-Tokens" imports Main begin text {* Proper proof text -- \<^bitalic>naive version\<^eitalic>. *} theorem and_comms: "\ \ \ \ \ \ \" proof assume "\ \ \" then show "\ \ \" proof assume "\" and "\" then show ?thesis .. qed qed text {* \<^bbold>Unstructured\<^ebold> proof script. *} theorem "\\<^isub>\ \ \\<^isub>\ \ \\<^isub>\ \ \\<^isub>\" apply (rule impI) apply (erule conjE) apply (rule conjI) apply assumption apply assumption done end