src/HOL/Complex_Main.thy
author wenzelm
Sun, 27 Oct 2024 12:32:40 +0100
changeset 81275 5ed639c16ce7
parent 80177 1478555580af
permissions -rw-r--r--
tuned;

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

theory Complex_Main
imports
  Complex
  MacLaurin
  Binomial_Plus
begin

end