# HG changeset patch # User immler # Date 1547685288 18000 # Node ID 56acd449da41acb13ce5e71ea4f01dbe037c2077 # Parent 880ab0f27ddf62cd666a9f557274b6ab32282968 chapters for analysis manual diff -r 880ab0f27ddf -r 56acd449da41 src/HOL/Analysis/Analysis.thy --- 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 diff -r 880ab0f27ddf -r 56acd449da41 src/HOL/Analysis/Elementary_Metric_Spaces.thy --- a/src/HOL/Analysis/Elementary_Metric_Spaces.thy Wed Jan 16 18:14:02 2019 -0500 +++ b/src/HOL/Analysis/Elementary_Metric_Spaces.thy Wed Jan 16 19:34:48 2019 -0500 @@ -4,13 +4,15 @@ Author: Brian Huffman, Portland State University *) -section \Elementary Metric Spaces\ +chapter \Functional Analysis\ theory Elementary_Metric_Spaces imports Abstract_Topology_2 begin +section \Elementary Metric Spaces\ + subsection \Open and closed balls\ definition%important ball :: "'a::metric_space \ real \ 'a set" diff -r 880ab0f27ddf -r 56acd449da41 src/HOL/Analysis/Elementary_Topology.thy --- a/src/HOL/Analysis/Elementary_Topology.thy Wed Jan 16 18:14:02 2019 -0500 +++ b/src/HOL/Analysis/Elementary_Topology.thy Wed Jan 16 19:34:48 2019 -0500 @@ -4,7 +4,7 @@ Author: Brian Huffman, Portland State University *) -section \Elementary Topology\ +chapter \Topology\ theory Elementary_Topology imports @@ -14,6 +14,8 @@ begin +section \Elementary Topology\ + subsection \TODO: move?\ lemma open_subopen: "open S \ (\x\S. \T. open T \ x \ T \ T \ S)" diff -r 880ab0f27ddf -r 56acd449da41 src/HOL/Analysis/L2_Norm.thy --- a/src/HOL/Analysis/L2_Norm.thy Wed Jan 16 18:14:02 2019 -0500 +++ b/src/HOL/Analysis/L2_Norm.thy Wed Jan 16 19:34:48 2019 -0500 @@ -2,12 +2,14 @@ Author: Brian Huffman, Portland State University *) -section \L2 Norm\ +chapter \Linear Algebra\ theory L2_Norm imports Complex_Main begin +section \L2 Norm\ + definition%important L2_set :: "('a \ real) \ 'a set \ real" where "L2_set f A = sqrt (\i\A. (f i)\<^sup>2)" diff -r 880ab0f27ddf -r 56acd449da41 src/HOL/Analysis/Sigma_Algebra.thy --- a/src/HOL/Analysis/Sigma_Algebra.thy Wed Jan 16 18:14:02 2019 -0500 +++ b/src/HOL/Analysis/Sigma_Algebra.thy Wed Jan 16 19:34:48 2019 -0500 @@ -5,7 +5,7 @@ translated by Lawrence Paulson. *) -section \Sigma Algebra\ +chapter \Measure and Integration Theory\ theory Sigma_Algebra imports @@ -17,6 +17,9 @@ "HOL-Library.Disjoint_Sets" begin + +section \Sigma Algebra\ + text \Sigma algebras are an elementary concept in measure theory. To measure --- that is to integrate --- functions, we first have to measure sets. Unfortunately, when dealing with a large universe, diff -r 880ab0f27ddf -r 56acd449da41 src/HOL/Analysis/Starlike.thy --- a/src/HOL/Analysis/Starlike.thy Wed Jan 16 18:14:02 2019 -0500 +++ b/src/HOL/Analysis/Starlike.thy Wed Jan 16 19:34:48 2019 -0500 @@ -5,13 +5,14 @@ Author: Armin Heller, TU Muenchen Author: Johannes Hoelzl, TU Muenchen *) - -section \Line Segments\ +chapter \Unsorted\ theory Starlike imports Convex_Euclidean_Space begin +section \Line Segments\ + subsection \Midpoint\ definition%important midpoint :: "'a::real_vector \ 'a \ 'a" diff -r 880ab0f27ddf -r 56acd449da41 src/HOL/Analysis/Topology_Euclidean_Space.thy --- a/src/HOL/Analysis/Topology_Euclidean_Space.thy Wed Jan 16 18:14:02 2019 -0500 +++ b/src/HOL/Analysis/Topology_Euclidean_Space.thy Wed Jan 16 19:34:48 2019 -0500 @@ -4,7 +4,7 @@ Author: Brian Huffman, Portland State University *) -section \Elementary Topology in Euclidean Space\ +chapter \Vector Analysis\ theory Topology_Euclidean_Space imports @@ -13,6 +13,8 @@ Norm_Arith begin +section \Elementary Topology in Euclidean Space\ + lemma euclidean_dist_l2: fixes x y :: "'a :: euclidean_space" shows "dist x y = L2_set (\i. dist (x \ i) (y \ i)) Basis" diff -r 880ab0f27ddf -r 56acd449da41 src/HOL/Analysis/document/root.tex --- a/src/HOL/Analysis/document/root.tex Wed Jan 16 18:14:02 2019 -0500 +++ b/src/HOL/Analysis/document/root.tex Wed Jan 16 19:34:48 2019 -0500 @@ -1,4 +1,4 @@ -\documentclass[11pt,a4paper]{article} +\documentclass[11pt,a4paper]{book} \usepackage{graphicx} \usepackage{isabelle} \usepackage{isabellesym}