| author | wenzelm | 
| Thu, 15 Aug 2019 16:57:09 +0200 | |
| changeset 70538 | fc9ba6fe367f | 
| parent 69605 | a96320074298 | 
| permissions | -rw-r--r-- | 
(* Title: HOL/Library/Adhoc_Overloading.thy Author: Alexander Krauss, TU Muenchen Author: Christian Sternagel, University of Innsbruck *) section \<open>Adhoc overloading of constants based on their types\<close> theory Adhoc_Overloading imports Main keywords "adhoc_overloading" "no_adhoc_overloading" :: thy_decl begin ML_file \<open>adhoc_overloading.ML\<close> end