src/Tools/Adhoc_Overloading.thy
author nipkow
Tue, 20 Sep 2011 05:47:11 +0200
changeset 45014 0e847655b2d8
parent 37818 dd65033fed78
child 48892 0b2407f406e8
permissions -rw-r--r--
New proof method "induction" that gives induction hypotheses the name IH.

(* Author: Alexander Krauss, TU Muenchen
   Author: Christian Sternagel, University of Innsbruck
*)

header {* Ad-hoc overloading of constants based on their types *}

theory Adhoc_Overloading
imports Pure
uses "adhoc_overloading.ML"
begin

setup Adhoc_Overloading.setup

end