src/HOL/Complex_Main.thy
author wenzelm
Mon, 04 Oct 2021 20:07:51 +0200
changeset 74449 a2dcda6107d9
parent 73411 1f1366966296
permissions -rw-r--r--
discontinued perl;

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

theory Complex_Main
imports
  Complex
  MacLaurin
begin

end