src/HOL/Complex_Analysis/Complex_Analysis.thy
author wenzelm
Tue, 25 Aug 2020 14:54:41 +0200
changeset 72205 bc71db05abe3
parent 71201 6617fb368a06
child 77277 c6b50597abbc
permissions -rw-r--r--
removed pointless version checks: Isabelle component integration does the job already;

theory Complex_Analysis
imports
  Residue_Theorem
  Riemann_Mapping
begin

end