src/Tools/Adhoc_Overloading.thy
author haftmann
Tue, 26 Jun 2012 22:09:34 +0200
changeset 48150 c97656ff4154
parent 37818 dd65033fed78
child 48892 0b2407f406e8
permissions -rw-r--r--
snippet to be sourced in user settings file in order to initialize components for a repository revision; the initialization is »liberal« since there is no obvious solution yet for components whose distribution is restricted

(* 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