src/Tools/Adhoc_Overloading.thy
author Lars Hupel <lars.hupel@mytum.de>
Mon, 19 May 2014 19:17:15 +0200
changeset 57004 c8288ce9676a
parent 52893 aa2afbafd983
child 58889 5b7a9633cfa8
permissions -rw-r--r--
trace windows uses search feature of Pretty_Text_Area; recursive invocations and intermediate steps are now shown in order; refinements to the exclusion of uninteresting subtraces in the output

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

header {* Adhoc overloading of constants based on their types *}

theory Adhoc_Overloading
imports Pure
keywords "adhoc_overloading" :: thy_decl and  "no_adhoc_overloading" :: thy_decl
begin

ML_file "adhoc_overloading.ML"

end