src/Tools/Adhoc_Overloading.thy
changeset 62020 5d208fd2507d
parent 58889 5b7a9633cfa8
child 63432 ba7901e94e7b
equal deleted inserted replaced
62019:9de1eb745aeb 62020:5d208fd2507d
     1 (* Author: Alexander Krauss, TU Muenchen
     1 (* Author: Alexander Krauss, TU Muenchen
     2    Author: Christian Sternagel, University of Innsbruck
     2    Author: Christian Sternagel, University of Innsbruck
     3 *)
     3 *)
     4 
     4 
     5 section {* Adhoc overloading of constants based on their types *}
     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 "adhoc_overloading" :: thy_decl and  "no_adhoc_overloading" :: thy_decl
    10 begin
    10 begin