| author | eberlm | 
| Fri, 17 Jun 2016 11:33:52 +0200 | |
| changeset 63319 | bc8793d7bd21 | 
| parent 62020 | 5d208fd2507d | 
| child 63432 | ba7901e94e7b | 
| permissions | -rw-r--r-- | 
| 37789 | 1  | 
(* Author: Alexander Krauss, TU Muenchen  | 
2  | 
Author: Christian Sternagel, University of Innsbruck  | 
|
3  | 
*)  | 
|
4  | 
||
| 62020 | 5  | 
section \<open>Adhoc overloading of constants based on their types\<close>  | 
| 37789 | 6  | 
|
7  | 
theory Adhoc_Overloading  | 
|
| 
37818
 
dd65033fed78
load cache_io before code generator; moved adhoc-overloading to generic tools
 
haftmann 
parents: 
37789 
diff
changeset
 | 
8  | 
imports Pure  | 
| 
52622
 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 
wenzelm 
parents: 
48892 
diff
changeset
 | 
9  | 
keywords "adhoc_overloading" :: thy_decl and "no_adhoc_overloading" :: thy_decl  | 
| 37789 | 10  | 
begin  | 
11  | 
||
| 48892 | 12  | 
ML_file "adhoc_overloading.ML"  | 
| 37789 | 13  | 
|
14  | 
end  | 
|
| 
37818
 
dd65033fed78
load cache_io before code generator; moved adhoc-overloading to generic tools
 
haftmann 
parents: 
37789 
diff
changeset
 | 
15  |