src/Tools/isac/Test.thy
branchisac-update-Isa09-2
changeset 37947 22235e4dbe5f
parent 37946 a28b5fc129b7
child 37948 ed85f172569c
     1.1 --- a/src/Tools/isac/Test.thy	Wed Aug 25 15:15:01 2010 +0200
     1.2 +++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
     1.3 @@ -1,7 +0,0 @@
     1.4 -theory Test imports Main begin;
     1.5 -   theorem my_thm: " A & B --> B & A";
     1.6 -   proof;
     1.7 -       assume " A & B";
     1.8 -       then obtain B and A ..;
     1.9 -       then show  "B & A" ..;
    1.10 -   qed;