src/Tools/Adhoc_Overloading.thy
changeset 63432 ba7901e94e7b
parent 62020 5d208fd2507d
equal deleted inserted replaced
63431:8002eec44fbb 63432:ba7901e94e7b
     4 
     4 
     5 section \<open>Adhoc overloading of constants based on their types\<close>
     5 section \<open>Adhoc overloading of constants based on their types\<close>
     6 
     6 
     7 theory Adhoc_Overloading
     7 theory Adhoc_Overloading
     8 imports Pure
     8 imports Pure
     9 keywords "adhoc_overloading" :: thy_decl and  "no_adhoc_overloading" :: thy_decl
     9 keywords
       
    10   "adhoc_overloading" "no_adhoc_overloading" :: thy_decl
    10 begin
    11 begin
    11 
    12 
    12 ML_file "adhoc_overloading.ML"
    13 ML_file "adhoc_overloading.ML"
    13 
    14 
    14 end
    15 end