src/HOL/Complex_Analysis/Complex_Analysis.thy
author wenzelm
Thu, 11 Apr 2024 12:05:01 +0200
changeset 80109 dbcd6dc7f70f
parent 79933 3f415c76a511
permissions -rw-r--r--
back to static numa_nodes (reverting part of c2c59de57df9);

theory Complex_Analysis
  imports
  Riemann_Mapping
  Residue_Theorem
  Weierstrass_Factorization
begin

end