author | wenzelm |
Wed, 16 Apr 2014 13:28:21 +0200 | |
changeset 56603 | 4f45570e532d |
parent 52893 | aa2afbafd983 |
child 58889 | 5b7a9633cfa8 |
permissions | -rw-r--r-- |
37789 | 1 |
(* Author: Alexander Krauss, TU Muenchen |
2 |
Author: Christian Sternagel, University of Innsbruck |
|
3 |
*) |
|
4 |
||
52893 | 5 |
header {* Adhoc overloading of constants based on their types *} |
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 |