src/HOL/Complex_Main.thy
author wenzelm
Sun, 27 May 2018 22:37:08 +0200
changeset 68300 cd8ab1a7a286
parent 63571 aee0d92995b6
child 73411 1f1366966296
permissions -rw-r--r--
retain isolated blob nodes (amending deb2fcbda16e): avoid failure of Session.handle_change with "Missing blob", when opening theory with load command later;

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

theory Complex_Main
imports
  Complex
  MacLaurin
begin

end