src/HOL/Complex_Main.thy
author immler
Tue, 12 Apr 2016 11:18:29 +0200
changeset 62949 f36a54da47a4
parent 60758 d8d85a8172b5
child 63570 1826a90b9cbc
permissions -rw-r--r--
added derivative of scaling in exponential function

section \<open>Comprehensive Complex Theory\<close>

theory Complex_Main
imports
  Main
  Real
  Complex
  Transcendental
  Taylor
  Deriv
begin

end