src/HOL/Complex_Main.thy
author paulson <lp15@cam.ac.uk>
Wed, 02 Apr 2014 16:45:31 +0100
changeset 56366 0362c3bb4d02
parent 51527 bd62e7ff103b
child 58889 5b7a9633cfa8
permissions -rw-r--r--
new theorem about zero limits

header {* Comprehensive Complex Theory *}

theory Complex_Main
imports
  Main
  Real
  Complex
  Transcendental
  Taylor
  Deriv
begin

end