src/Tools/Adhoc_Overloading.thy
author blanchet
Wed, 05 Jun 2013 13:19:26 +0200
changeset 52303 16d7708aba40
parent 48892 0b2407f406e8
child 52622 e0ff1625e96d
permissions -rw-r--r--
one less flaky "fpTs" check (flaky in the presence of duplicates in "fpTs", which we want to have in "primrec")

(* 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
begin

ML_file "adhoc_overloading.ML"
setup Adhoc_Overloading.setup

end