src/HOL/Complex_Main.thy
author paulson
Fri, 17 Mar 2023 10:42:50 +0000
changeset 77685 05329cd9db4b
parent 73411 1f1366966296
child 80177 1478555580af
permissions -rw-r--r--
merged

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

theory Complex_Main
imports
  Complex
  MacLaurin
begin

end