make this module appeat late in Pure;
moved print_current_goals to display.ML;
added quick_and_dirty_prove_goalw_cterm (from Isar/skip_proof.ML);
added thm database functions (from Thy/thm_database.ML);
(* Title: HOLCF/Lift2.thy
ID: $Id$
Author: Olaf Mueller
Copyright 1996 Technische Universitaet Muenchen
Class Instance lift::(term)po
*)
Lift2 = Lift1 +
instance "lift" :: (term)po (refl_less_lift,antisym_less_lift,trans_less_lift)
end