src/HOL/Complex_Analysis/Complex_Analysis.thy
author wenzelm
Tue, 28 Sep 2021 22:50:22 +0200
changeset 74386 40804452ab6b
parent 71201 6617fb368a06
child 77277 c6b50597abbc
permissions -rw-r--r--
recover some Linux test, using virtual machine node (Ubuntu 20.04, 4 cores, 16 GB);

theory Complex_Analysis
imports
  Residue_Theorem
  Riemann_Mapping
begin

end