src/HOL/Complex_Main.thy
author Manuel Eberl <manuel@pruvisto.org>
Tue, 15 Apr 2025 17:38:20 +0200
changeset 82518 da14e77a48b2
parent 80177 1478555580af
permissions -rw-r--r--
lots of lemmas for HOL, HOL-{Complex_}Analysis, HOL-Number_Theory

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

theory Complex_Main
imports
  Complex
  MacLaurin
  Binomial_Plus
begin

end