src/Tools/isac/Test.thy
author Walther Neuper <neuper@ist.tugraz.at>
Thu, 19 Aug 2010 12:08:42 +0200
branchisac-update-Isa09-2
changeset 37929 862f35fdb091
parent 37906 e2b23ba9df13
permissions -rw-r--r--
reduced ctxt_Isac and ctxt_HOL to fun thy2ctxt', thy2ctxt
     1 theory Test imports Main begin;
     2    theorem my_thm: " A & B --> B & A";
     3    proof;
     4        assume " A & B";
     5        then obtain B and A ..;
     6        then show  "B & A" ..;
     7    qed;