src/HOL/Complex_Main.thy
author wenzelm
Tue, 12 Jan 2010 22:23:29 +0100
changeset 34882 7ad1189d54ca
parent 33269 3b7e2dbbd684
child 35292 e4a431b6d9b7
permissions -rw-r--r--
rebuilt from fresh copy of Bitstream Vera, for improved quality of regular text glyphs; misc cleanup of mathematical glyphs, with bold version synthesized by fontforge;

header {* Comprehensive Complex Theory *}

theory Complex_Main
imports
  Main
  Real
  SupInf
  Complex
  Log
  Ln
  Taylor
  Integration
begin

end