src/HOL/Complex_Analysis/Complex_Analysis.thy
author Fabian Huch <huch@in.tum.de>
Wed, 08 Nov 2023 11:08:03 +0100
changeset 78928 6c2c60b852e0
parent 77277 c6b50597abbc
child 79875 0e9a809dc0b2
permissions -rw-r--r--
move timing data into scheduler for more efficient heuristics (e.g., with pre-calculated values);
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
71189
954ee5acaae0 Split off new HOL-Complex_Analysis session from HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
     1
theory Complex_Analysis
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents: 71189
diff changeset
     2
imports
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents: 71189
diff changeset
     3
  Residue_Theorem
77277
c6b50597abbc More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents: 71201
diff changeset
     4
  Meromorphic
71189
954ee5acaae0 Split off new HOL-Complex_Analysis session from HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
     5
begin
954ee5acaae0 Split off new HOL-Complex_Analysis session from HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
     6
954ee5acaae0 Split off new HOL-Complex_Analysis session from HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
     7
end