CookBook/Recipes/Transformation.thy
author Christian Urban <urbanc@in.tum.de>
Thu, 12 Feb 2009 16:09:42 +0000
changeset 110 12533bb49615
parent 13 2b07da8b310d
permissions -rw-r--r--
recovered old version of simple_induct; split the main function into small functions


theory Transformation
imports Main
begin


section {* Ad-hoc Transformations of Theorems *}



end