src/HOL/Complex_Main.thy
author wenzelm
Sun, 03 Jan 2016 21:45:34 +0100
changeset 62048 fefd79f6b232
parent 60758 d8d85a8172b5
child 63570 1826a90b9cbc
permissions -rw-r--r--
retain ASCII syntax for output, when HOL/Library/Lattice_Syntax is not present (amending e96292f32c3c);

section \<open>Comprehensive Complex Theory\<close>

theory Complex_Main
imports
  Main
  Real
  Complex
  Transcendental
  Taylor
  Deriv
begin

end