src/HOL/Complex_Main.thy
author haftmann
Mon, 29 Dec 2008 14:08:08 +0100
changeset 29197 6d4cb27ed19c
parent 29026 5fbaa05f637f
child 29304 5c71a6da989d
permissions -rw-r--r--
adapted HOL source structure to distribution layout

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

header{*Comprehensive Complex Theory*}

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

end