src/Tools/Adhoc_Overloading.thy
author wenzelm
Sat, 23 May 2015 17:19:37 +0200
changeset 60299 5ae2a2e74c93
parent 58889 5b7a9633cfa8
child 62020 5d208fd2507d
permissions -rw-r--r--
clarified NEWS: document_files are officially required since Isabelle2014, but the absence was tolerated as legacy feature;

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

section {* 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