make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
(* Title: HOL/ex/Interpretation_with_Defs.thy
Author: Florian Haftmann, TU Muenchen
*)
header {* Interpretation accompanied with mixin definitions. EXPERIMENTAL. *}
theory Interpretation_with_Defs
imports Pure
begin
ML_file "~~/src/Tools/interpretation_with_defs.ML"
end