src/HOL/Complex_Main.thy
author nipkow
Sun, 15 Feb 2009 16:25:16 +0100
changeset 29923 24f56736c56f
parent 29879 4425849f5db7
child 29986 6b1ccda8bf19
permissions -rw-r--r--
added finite_set_choice

header {* Comprehensive Complex Theory *}

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

end