src/HOL/Complex_Main.thy
author popescua
Fri, 24 May 2013 19:09:56 +0200
changeset 52183 667961fa6a60
parent 51527 bd62e7ff103b
child 58889 5b7a9633cfa8
permissions -rw-r--r--
fixed files broken due to Zorn changes (cf. 59e5dd7b8f9a)

header {* Comprehensive Complex Theory *}

theory Complex_Main
imports
  Main
  Real
  Complex
  Transcendental
  Taylor
  Deriv
begin

end