make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
(* Title: HOL/HOLCF/Plain_HOLCF.thy
Author: Brian Huffman
*)
header {* Plain HOLCF *}
theory Plain_HOLCF
imports Cfun Sfun Cprod Sprod Ssum Up Discrete Lift One Tr Fix
begin
text {*
Basic HOLCF concepts and types; does not include definition packages.
*}
end