added option quickcheck_locale to allow different behaviours for handling locales in Quickcheck;
added examples of quickcheck_locale option;
trying to speed up Quickcheck_Examples;
(* 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