src/HOL/Analysis/Analysis.thy
author wenzelm
Wed, 07 Mar 2018 17:27:57 +0100
changeset 67778 a25f9076a0b3
parent 67727 ce3e87a51488
child 67996 6a9d1b31a7c5
permissions -rw-r--r--
eliminated somewhat pointless parallelism (from 857da80611ab): usually hundreds of tasks with < 1ms each, also note that the enclosing join_theory happens within theory graph parallelism;

theory Analysis
imports
  Lebesgue_Integral_Substitution
  Improper_Integral
  Embed_Measure
  Complete_Measure
  Radon_Nikodym
  Fashoda_Theorem
  Determinants
  Homeomorphism
  Bounded_Continuous_Function
  Function_Topology
  Infinite_Products
  Infinite_Set_Sum
  Weierstrass_Theorems
  Polytope
  Jordan_Curve
  Winding_Numbers
  Riemann_Mapping
  Poly_Roots
  Conformal_Mappings
  FPS_Convergence
  Generalised_Binomial_Theorem
  Gamma_Function
  Ball_Volume
  Lipschitz
begin

end