added Induct/Binary_Trees.thy, Induct/Datatypes.thy;
removed ex/Data.ML ex/Data.thy ex/Enum.ML ex/Enum.thy;
(* Title: HOLCF/Fun3.thy
ID: $Id$
Author: Franz Regensburger
License: GPL (GNU GENERAL PUBLIC LICENSE)
Class instance of => (fun) for class pcpo
*)
Fun3 = Fun2 +
(* default class is still term *)
instance fun :: (term,cpo)cpo (cpo_fun)
instance fun :: (term,pcpo)pcpo (least_fun)
end