src/HOL/Complex_Analysis/Complex_Analysis.thy
author wenzelm
Wed, 13 Aug 2025 19:40:09 +0200
changeset 83005 a2a860cd3215
parent 79933 3f415c76a511
permissions -rw-r--r--
more robust, notably for Isabelle/MAWEN "polyminus.sml matchsub (?a * (?b - ?c)...";

theory Complex_Analysis
  imports
  Riemann_Mapping
  Residue_Theorem
  Weierstrass_Factorization
begin

end