changeset 68061 | 81d90f830f99 |
parent 68060 | 3931ed905e93 |
child 68063 | 539048827fe8 |
--- a/src/Tools/Adhoc_Overloading.thy Tue May 01 16:42:14 2018 +0200 +++ /dev/null Thu Jan 01 00:00:00 1970 +0000 @@ -1,16 +0,0 @@ -(* 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 Pure -keywords - "adhoc_overloading" "no_adhoc_overloading" :: thy_decl -begin - -ML_file "adhoc_overloading.ML" - -end -