src/HOL/Complex_Analysis/Complex_Analysis.thy
author wenzelm
Wed, 14 Feb 2024 14:41:18 +0100
changeset 79604 0e8ac7db1f4d
parent 77277 c6b50597abbc
child 79875 0e9a809dc0b2
permissions -rw-r--r--
clarified num_processors: follow Poly/ML (with its inaccuracies);

theory Complex_Analysis
imports
  Residue_Theorem
  Meromorphic
begin

end