make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
(* Title: HOL/Import/HOL_Light_Import.thy
Author: Cezary Kaliszyk, University of Innsbruck
Author: Alexander Krauss, QAware GmbH
*)
header {* Main HOL Light importer *}
theory HOL_Light_Import
imports HOL_Light_Maps
begin
import_file "$HOL_LIGHT_BUNDLE"
end