replaced low-level Term.str_of by Display.raw_string_of_term (should actually use Display.string_of_term);
(* Title: HOL/Complex/Complex_Main.thy
ID: $Id$
Author: Lawrence C Paulson, Cambridge University Computer Laboratory
Copyright 2003 University of Cambridge
*)
header{*Comprehensive Complex Theory*}
theory Complex_Main
imports CLim
begin
end