src/Tools/Adhoc_Overloading.thy
changeset 37818 dd65033fed78
parent 37789 93f6dcf9ec02
child 48892 0b2407f406e8
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/Tools/Adhoc_Overloading.thy	Wed Jul 14 14:16:12 2010 +0200
@@ -0,0 +1,15 @@
+(* Author: Alexander Krauss, TU Muenchen
+   Author: Christian Sternagel, University of Innsbruck
+*)
+
+header {* Ad-hoc overloading of constants based on their types *}
+
+theory Adhoc_Overloading
+imports Pure
+uses "adhoc_overloading.ML"
+begin
+
+setup Adhoc_Overloading.setup
+
+end
+