src/HOL/Library/Adhoc_Overloading.thy
changeset 68061 81d90f830f99
parent 63432 ba7901e94e7b
child 69605 a96320074298
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Library/Adhoc_Overloading.thy	Tue May 01 20:40:27 2018 +0200
@@ -0,0 +1,15 @@
+(*  Title:      HOL/Library/Adhoc_Overloading.thy
+    Author:     Alexander Krauss, TU Muenchen
+    Author:     Christian Sternagel, University of Innsbruck
+*)
+
+section \<open>Adhoc overloading of constants based on their types\<close>
+
+theory Adhoc_Overloading
+  imports Main
+  keywords "adhoc_overloading" "no_adhoc_overloading" :: thy_decl
+begin
+
+ML_file "adhoc_overloading.ML"
+
+end