src/HOL/Complex_Main.thy
author haftmann
Wed, 21 Jan 2009 16:47:31 +0100
changeset 29580 117b88da143c
parent 29304 5c71a6da989d
child 29879 4425849f5db7
permissions -rw-r--r--
dropped ID

header {* Comprehensive Complex Theory *}

theory Complex_Main
imports
  Main
  Real
  Fundamental_Theorem_Algebra
  Log
  Ln
  Taylor
  Integration
  FrechetDeriv
begin

end