src/HOL/Analysis/Analysis.thy
changeset 69676 56acd449da41
parent 69144 f13b82281715
child 69874 11065b70407d
--- a/src/HOL/Analysis/Analysis.thy	Wed Jan 16 18:14:02 2019 -0500
+++ b/src/HOL/Analysis/Analysis.thy	Wed Jan 16 19:34:48 2019 -0500
@@ -1,5 +1,20 @@
 theory Analysis
-imports
+  imports
+  (* Linear Algebra *)
+  Convex
+  Determinants
+  (* Topology *)
+  Connected
+  (* Functional Analysis *)
+  Elementary_Normed_Spaces
+  Norm_Arith
+  (* Vector Analysis *)
+  Convex_Euclidean_Space
+  (* Measure and Integration Theory *)
+  Ball_Volume
+  Integral_Test
+  Improper_Integral
+  (* Unsorted *)
   Lebesgue_Integral_Substitution
   Improper_Integral
   Embed_Measure