src/HOL/Complex_Main.thy
author wenzelm
Mon, 22 Sep 2025 15:55:47 +0200
changeset 83211 1d189ef55adf
parent 80177 1478555580af
permissions -rw-r--r--
more accurate markup for command timing, notably for theory pseudo-command in batch-build, but also for accidental occurrences of command keywords (e.g. in command definition);

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

theory Complex_Main
imports
  Complex
  MacLaurin
  Binomial_Plus
begin

end