src/HOL/Complex_Main.thy
author huffman
Wed, 03 Jun 2009 07:44:56 -0700
changeset 31413 729d90a531e4
parent 31204 46c0c741c8c2
child 33269 3b7e2dbbd684
permissions -rw-r--r--
introduce class topological_space as a superclass of metric_space

header {* Comprehensive Complex Theory *}

theory Complex_Main
imports
  Main
  Real
  Complex
  Log
  Ln
  Taylor
  Integration
begin

end