src/HOL/Complex/Complex_Main.thy
author huffman
Thu, 03 Jul 2008 18:16:40 +0200
changeset 27475 61b979a2c820
parent 27472 47bc28e011d5
child 27541 9e585e99b494
permissions -rw-r--r--
add Infinite_Set and Zorn back in (since they are no longer included in main HOL image)

(*  Title:      HOL/Complex/Complex_Main.thy
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   2003  University of Cambridge
*)

header{*Comprehensive Complex Theory*}

theory Complex_Main
imports
  Main
  Fundamental_Theorem_Algebra
  "../Hyperreal/Log"
  "../Hyperreal/Ln"
  "../Hyperreal/Taylor"
  "../Hyperreal/Integration"
begin

end