src/Tools/Adhoc_Overloading.thy
changeset 52893 aa2afbafd983
parent 52622 e0ff1625e96d
child 58889 5b7a9633cfa8
equal deleted inserted replaced
52892:9ce4d52c9176 52893:aa2afbafd983
     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 header {* Ad-hoc overloading of constants based on their types *}
     5 header {* Adhoc overloading of constants based on their types *}
     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