src/HOL/Complex_Main.thy
author haftmann
Wed, 25 Dec 2013 15:52:25 +0100
changeset 54861 00d551179872
parent 51527 bd62e7ff103b
child 58889 5b7a9633cfa8
permissions -rw-r--r--
postponed min/max lemmas until abstract lattice is available

header {* Comprehensive Complex Theory *}

theory Complex_Main
imports
  Main
  Real
  Complex
  Transcendental
  Taylor
  Deriv
begin

end