src/HOL/Complex_Main.thy
author wenzelm
Fri, 07 May 2021 13:17:29 +0200
changeset 73642 ac6f8fff036b
parent 73411 1f1366966296
child 80177 1478555580af
permissions -rw-r--r--
clarified default_platform_families (again);

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

theory Complex_Main
imports
  Complex
  MacLaurin
begin

end