src/Tools/Adhoc_Overloading.thy
changeset 68061 81d90f830f99
parent 68060 3931ed905e93
child 68063 539048827fe8
equal deleted inserted replaced
68060:3931ed905e93 68061:81d90f830f99
     1 (* Author: Alexander Krauss, TU Muenchen
       
     2    Author: Christian Sternagel, University of Innsbruck
       
     3 *)
       
     4 
       
     5 section \<open>Adhoc overloading of constants based on their types\<close>
       
     6 
       
     7 theory Adhoc_Overloading
       
     8 imports Pure
       
     9 keywords
       
    10   "adhoc_overloading" "no_adhoc_overloading" :: thy_decl
       
    11 begin
       
    12 
       
    13 ML_file "adhoc_overloading.ML"
       
    14 
       
    15 end
       
    16