src/HOL/Complex_Main.thy
author wenzelm
Thu, 19 Dec 2019 15:29:48 +0100
changeset 71318 1be996d8bb98
parent 63571 aee0d92995b6
child 73411 1f1366966296
permissions -rw-r--r--
proper proof body context for Simplifier plugins (solvers, loopers, ...) -- avoid crash due to Subgoal.FOCUS (before e58bc223f46c);

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

theory Complex_Main
imports
  Complex
  MacLaurin
begin

end