# HG changeset patch # User wenzelm # Date 1446460982 -3600 # Node ID f92bf6674699fce4ae45c65c5aafd499488c2649 # Parent a29295dac1ca8425b072bfd03bef59405d0d39c9 tuned document; diff -r a29295dac1ca -r f92bf6674699 src/HOL/Hahn_Banach/Function_Norm.thy --- a/src/HOL/Hahn_Banach/Function_Norm.thy Mon Nov 02 11:10:28 2015 +0100 +++ b/src/HOL/Hahn_Banach/Function_Norm.thy Mon Nov 02 11:43:02 2015 +0100 @@ -11,14 +11,13 @@ subsection \Continuous linear forms\ text \ - A linear form \f\ on a normed vector space \(V, \\\)\ - is \<^emph>\continuous\, iff it is bounded, i.e. + A linear form \f\ on a normed vector space \(V, \\\)\ is \<^emph>\continuous\, + iff it is bounded, i.e. \begin{center} \\c \ R. \x \ V. \f x\ \ c \ \x\\ \end{center} - In our application no other functions than linear forms are - considered, so we can define continuous linear forms as bounded - linear forms: + In our application no other functions than linear forms are considered, so + we can define continuous linear forms as bounded linear forms: \ locale continuous = linearform + @@ -48,28 +47,25 @@ \end{center} is called the \<^emph>\norm\ of \f\. - For non-trivial vector spaces \V \ {0}\ the norm can be - defined as + For non-trivial vector spaces \V \ {0}\ the norm can be defined as \begin{center} \\f\ = \x \ 0. \f x\ / \x\\ \end{center} - For the case \V = {0}\ the supremum would be taken from an - empty set. Since \\\ is unbounded, there would be no supremum. - To avoid this situation it must be guaranteed that there is an - element in this set. This element must be \{} \ 0\ so that - \fn_norm\ has the norm properties. Furthermore it does not - have to change the norm in all other cases, so it must be \0\, - as all other elements are \{} \ 0\. + For the case \V = {0}\ the supremum would be taken from an empty set. + Since \\\ is unbounded, there would be no supremum. To avoid this + situation it must be guaranteed that there is an element in this set. This + element must be \{} \ 0\ so that \fn_norm\ has the norm properties. + Furthermore it does not have to change the norm in all other cases, so it + must be \0\, as all other elements are \{} \ 0\. - Thus we define the set \B\ where the supremum is taken from as - follows: + Thus we define the set \B\ where the supremum is taken from as follows: \begin{center} \{0} \ {\f x\ / \x\. x \ 0 \ x \ F}\ \end{center} - \fn_norm\ is equal to the supremum of \B\, if the - supremum exists (otherwise it is undefined). + \fn_norm\ is equal to the supremum of \B\, if the supremum exists + (otherwise it is undefined). \ locale fn_norm = @@ -84,8 +80,8 @@ by (simp add: B_def) text \ - The following lemma states that every continuous linear form on a - normed space \(V, \\\)\ has a function norm. + The following lemma states that every continuous linear form on a normed + space \(V, \\\)\ has a function norm. \ lemma (in normed_vectorspace_with_fn_norm) fn_norm_works: @@ -108,9 +104,9 @@ txt \We know that \f\ is bounded by some value \c\.\ from bounded obtain c where c: "\x \ V. \f x\ \ c * \x\" .. - txt \To prove the thesis, we have to show that there is some - \b\, such that \y \ b\ for all \y \ - B\. Due to the definition of \B\ there are two cases.\ + txt \To prove the thesis, we have to show that there is some \b\, such + that \y \ b\ for all \y \ B\. Due to the definition of \B\ there are + two cases.\ def b \ "max c 0" have "\y \ B V f. y \ b" @@ -237,8 +233,8 @@ text \ \<^medskip> - The function norm is the least positive real number for - which the following inequation holds: + The function norm is the least positive real number for which the + following inequality holds: \begin{center} \\f x\ \ c \ \x\\ \end{center} diff -r a29295dac1ca -r f92bf6674699 src/HOL/Hahn_Banach/Function_Order.thy --- a/src/HOL/Hahn_Banach/Function_Order.thy Mon Nov 02 11:10:28 2015 +0100 +++ b/src/HOL/Hahn_Banach/Function_Order.thy Mon Nov 02 11:43:02 2015 +0100 @@ -70,8 +70,8 @@ where "funct g = (\x. (SOME y. (x, y) \ g))" text \ - The following lemma states that \g\ is the graph of a function - if the relation induced by \g\ is unique. + The following lemma states that \g\ is the graph of a function if the + relation induced by \g\ is unique. \ lemma graph_domain_funct: @@ -93,9 +93,9 @@ subsection \Norm-preserving extensions of a function\ text \ - Given a linear form \f\ on the space \F\ and a seminorm - \p\ on \E\. The set of all linear extensions of \f\, to superspaces \H\ of \F\, which are bounded by - \p\, is defined as follows. + Given a linear form \f\ on the space \F\ and a seminorm \p\ on \E\. The + set of all linear extensions of \f\, to superspaces \H\ of \F\, which are + bounded by \p\, is defined as follows. \ definition diff -r a29295dac1ca -r f92bf6674699 src/HOL/Hahn_Banach/Hahn_Banach.thy --- a/src/HOL/Hahn_Banach/Hahn_Banach.thy Mon Nov 02 11:10:28 2015 +0100 +++ b/src/HOL/Hahn_Banach/Hahn_Banach.thy Mon Nov 02 11:43:02 2015 +0100 @@ -9,37 +9,36 @@ begin text \ - We present the proof of two different versions of the Hahn-Banach - Theorem, closely following @{cite \\S36\ "Heuser:1986"}. + We present the proof of two different versions of the Hahn-Banach Theorem, + closely following @{cite \\S36\ "Heuser:1986"}. \ + subsection \The Hahn-Banach Theorem for vector spaces\ paragraph \Hahn-Banach Theorem.\ text \ - Let \F\ be a subspace of a real vector space \E\, let \p\ be a semi-norm on \E\, and \f\ be a linear form defined on - \F\ such that \f\ is bounded by \p\, i.e. \\x \ - F. f x \ p x\. Then \f\ can be extended to a linear form \h\ - on \E\ such that \h\ is norm-preserving, i.e. \h\ is - also bounded by \p\. -\ + Let \F\ be a subspace of a real vector space \E\, let \p\ be a semi-norm + on \E\, and \f\ be a linear form defined on \F\ such that \f\ is bounded + by \p\, i.e. \\x \ F. f x \ p x\. Then \f\ can be extended to a linear + form \h\ on \E\ such that \h\ is norm-preserving, i.e. \h\ is also bounded + by \p\. \ paragraph \Proof Sketch.\ text \ - \<^enum> Define \M\ as the set of norm-preserving extensions of - \f\ to subspaces of \E\. The linear forms in \M\ - are ordered by domain extension. + \<^enum> Define \M\ as the set of norm-preserving extensions of \f\ to subspaces + of \E\. The linear forms in \M\ are ordered by domain extension. - \<^enum> We show that every non-empty chain in \M\ has an upper - bound in \M\. + \<^enum> We show that every non-empty chain in \M\ has an upper bound in \M\. - \<^enum> With Zorn's Lemma we conclude that there is a maximal function - \g\ in \M\. + \<^enum> With Zorn's Lemma we conclude that there is a maximal function \g\ in + \M\. - \<^enum> The domain \H\ of \g\ is the whole space \E\, as shown by classical contradiction: + \<^enum> The domain \H\ of \g\ is the whole space \E\, as shown by classical + contradiction: - \<^item> Assuming \g\ is not defined on whole \E\, it can - still be extended in a norm-preserving way to a super-space \H'\ of \H\. + \<^item> Assuming \g\ is not defined on whole \E\, it can still be extended in + a norm-preserving way to a super-space \H'\ of \H\. \<^item> Thus \g\ can not be maximal. Contradiction! \ @@ -153,7 +152,7 @@ obtain xi where xi: "\y \ H. - p (y + x') - h y \ xi \ xi \ p (y + x') - h y" - -- \Pick a real number \\\ that fulfills certain inequations; this will\ + -- \Pick a real number \\\ that fulfills certain inequality; this will\ -- \be used to establish that \h'\ is a norm-preserving extension of \h\. \label{ex-xi-use}\<^smallskip>\ proof - @@ -292,10 +291,10 @@ text \ The following alternative formulation of the Hahn-Banach - Theorem\label{abs-Hahn-Banach} uses the fact that for a real linear - form \f\ and a seminorm \p\ the following inequations - are equivalent:\footnote{This was shown in lemma @{thm [source] - abs_ineq_iff} (see page \pageref{abs-ineq-iff}).} + Theorem\label{abs-Hahn-Banach} uses the fact that for a real linear form + \f\ and a seminorm \p\ the following inequality are + equivalent:\footnote{This was shown in lemma @{thm [source] abs_ineq_iff} + (see page \pageref{abs-ineq-iff}).} \begin{center} \begin{tabular}{lll} \\x \ H. \h x\ \ p x\ & and & @@ -336,9 +335,9 @@ subsection \The Hahn-Banach Theorem for normed spaces\ text \ - Every continuous linear form \f\ on a subspace \F\ of a - norm space \E\, can be extended to a continuous linear form - \g\ on \E\ such that \\f\ = \g\\. + Every continuous linear form \f\ on a subspace \F\ of a norm space \E\, + can be extended to a continuous linear form \g\ on \E\ such that \\f\ = + \g\\. \ theorem norm_Hahn_Banach: @@ -420,10 +419,10 @@ OF F_norm, folded B_def fn_norm_def]) qed - txt \Using the fact that \p\ is a seminorm and \f\ is bounded - by \p\ we can apply the Hahn-Banach Theorem for real vector - spaces. So \f\ can be extended in a norm-preserving way to - some function \g\ on the whole vector space \E\.\ + txt \Using the fact that \p\ is a seminorm and \f\ is bounded by \p\ we + can apply the Hahn-Banach Theorem for real vector spaces. So \f\ can be + extended in a norm-preserving way to some function \g\ on the whole + vector space \E\.\ with E FE linearform q obtain g where linearformE: "linearform E g" @@ -445,19 +444,20 @@ have "\g\\E = \f\\F" proof (rule order_antisym) txt \ - First we show \\g\ \ \f\\. The function norm \\g\\ is defined as the smallest \c \ \\ such that + First we show \\g\ \ \f\\. The function norm \\g\\ is defined as the + smallest \c \ \\ such that \begin{center} \begin{tabular}{l} \\x \ E. \g x\ \ c \ \x\\ \end{tabular} \end{center} - \noindent Furthermore holds + \<^noindent> Furthermore holds \begin{center} \begin{tabular}{l} \\x \ E. \g x\ \ \f\ \ \x\\ \end{tabular} \end{center} -\ + \ from g_cont _ ge_zero show "\g\\E \ \f\\F" diff -r a29295dac1ca -r f92bf6674699 src/HOL/Hahn_Banach/Hahn_Banach_Ext_Lemmas.thy --- a/src/HOL/Hahn_Banach/Hahn_Banach_Ext_Lemmas.thy Mon Nov 02 11:10:28 2015 +0100 +++ b/src/HOL/Hahn_Banach/Hahn_Banach_Ext_Lemmas.thy Mon Nov 02 11:43:02 2015 +0100 @@ -9,29 +9,27 @@ begin text \ - In this section the following context is presumed. Let \E\ be - a real vector space with a seminorm \q\ on \E\. \F\ is a subspace of \E\ and \f\ a linear function on - \F\. We consider a subspace \H\ of \E\ that is a - superspace of \F\ and a linear form \h\ on \H\. \H\ is a not equal to \E\ and \x\<^sub>0\ is - an element in \E - H\. \H\ is extended to the direct - sum \H' = H + lin x\<^sub>0\, so for any \x \ H'\ - the decomposition of \x = y + a \ x\ with \y \ H\ is - unique. \h'\ is defined on \H'\ by \h' x = h y + - a \ \\ for a certain \\\. + In this section the following context is presumed. Let \E\ be a real + vector space with a seminorm \q\ on \E\. \F\ is a subspace of \E\ and \f\ + a linear function on \F\. We consider a subspace \H\ of \E\ that is a + superspace of \F\ and a linear form \h\ on \H\. \H\ is a not equal to \E\ + and \x\<^sub>0\ is an element in \E - H\. \H\ is extended to the direct sum \H' + = H + lin x\<^sub>0\, so for any \x \ H'\ the decomposition of \x = y + a \ x\ + with \y \ H\ is unique. \h'\ is defined on \H'\ by \h' x = h y + a \ \\ + for a certain \\\. - Subsequently we show some properties of this extension \h'\ of - \h\. + Subsequently we show some properties of this extension \h'\ of \h\. \<^medskip> - This lemma will be used to show the existence of a linear - extension of \f\ (see page \pageref{ex-xi-use}). It is a - consequence of the completeness of \\\. To show + This lemma will be used to show the existence of a linear extension of \f\ + (see page \pageref{ex-xi-use}). It is a consequence of the completeness of + \\\. To show \begin{center} \begin{tabular}{l} \\\. \y \ F. a y \ \ \ \ \ b y\ \end{tabular} \end{center} - \noindent it suffices to show that + \<^noindent> it suffices to show that \begin{center} \begin{tabular}{l} \\u \ F. \v \ F. a u \ b v\ @@ -84,9 +82,8 @@ text \ \<^medskip> - The function \h'\ is defined as a \h' x = h y - + a \ \\ where \x = y + a \ \\ is a linear extension of - \h\ to \H'\. + The function \h'\ is defined as a \h' x = h y + a \ \\ where + \x = y + a \ \\ is a linear extension of \h\ to \H'\. \ lemma h'_lf: @@ -192,8 +189,8 @@ text \ \<^medskip> - The linear extension \h'\ of \h\ - is bounded by the seminorm \p\.\ + The linear extension \h'\ of \h\ is bounded by the seminorm \p\. +\ lemma h'_norm_pres: assumes h'_def: "h' \ \x. let (y, a) = diff -r a29295dac1ca -r f92bf6674699 src/HOL/Hahn_Banach/Hahn_Banach_Sup_Lemmas.thy --- a/src/HOL/Hahn_Banach/Hahn_Banach_Sup_Lemmas.thy Mon Nov 02 11:10:28 2015 +0100 +++ b/src/HOL/Hahn_Banach/Hahn_Banach_Sup_Lemmas.thy Mon Nov 02 11:43:02 2015 +0100 @@ -2,27 +2,25 @@ Author: Gertrud Bauer, TU Munich *) -section \The supremum w.r.t.~the function order\ +section \The supremum wrt.\ the function order\ theory Hahn_Banach_Sup_Lemmas imports Function_Norm Zorn_Lemma begin text \ - This section contains some lemmas that will be used in the proof of - the Hahn-Banach Theorem. In this section the following context is - presumed. Let \E\ be a real vector space with a seminorm - \p\ on \E\. \F\ is a subspace of \E\ and - \f\ a linear form on \F\. We consider a chain \c\ - of norm-preserving extensions of \f\, such that \\c = - graph H h\. We will show some properties about the limit function - \h\, i.e.\ the supremum of the chain \c\. + This section contains some lemmas that will be used in the proof of the + Hahn-Banach Theorem. In this section the following context is presumed. + Let \E\ be a real vector space with a seminorm \p\ on \E\. \F\ is a + subspace of \E\ and \f\ a linear form on \F\. We consider a chain \c\ of + norm-preserving extensions of \f\, such that \\c = graph H h\. We will + show some properties about the limit function \h\, i.e.\ the supremum of + the chain \c\. \<^medskip> - Let \c\ be a chain of norm-preserving extensions of - the function \f\ and let \graph H h\ be the supremum - of \c\. Every element in \H\ is member of one of the - elements of the chain. + Let \c\ be a chain of norm-preserving extensions of the function \f\ and + let \graph H h\ be the supremum of \c\. Every element in \H\ is member of + one of the elements of the chain. \ lemmas [dest?] = chainsD @@ -57,10 +55,10 @@ text \ \<^medskip> - Let \c\ be a chain of norm-preserving extensions of - the function \f\ and let \graph H h\ be the supremum - of \c\. Every element in the domain \H\ of the supremum - function is member of the domain \H'\ of some function \h'\, such that \h\ extends \h'\. + Let \c\ be a chain of norm-preserving extensions of the function \f\ and + let \graph H h\ be the supremum of \c\. Every element in the domain \H\ of + the supremum function is member of the domain \H'\ of some function \h'\, + such that \h\ extends \h'\. \ lemma some_H'h': @@ -85,10 +83,9 @@ text \ \<^medskip> - Any two elements \x\ and \y\ in the domain - \H\ of the supremum function \h\ are both in the domain - \H'\ of some function \h'\, such that \h\ extends - \h'\. + Any two elements \x\ and \y\ in the domain \H\ of the supremum function + \h\ are both in the domain \H'\ of some function \h'\, such that \h\ + extends \h'\. \ lemma some_H'h'2: @@ -158,8 +155,8 @@ text \ \<^medskip> - The relation induced by the graph of the supremum of a - chain \c\ is definite, i.~e.~t is the graph of a function. + The relation induced by the graph of the supremum of a chain \c\ is + definite, i.e.\ it is the graph of a function. \ lemma sup_definite: @@ -181,8 +178,8 @@ then obtain H2 h2 where G2_rep: "G2 = graph H2 h2" unfolding M_def by blast - txt \\G\<^sub>1\ is contained in \G\<^sub>2\ - or vice versa, since both \G\<^sub>1\ and \G\<^sub>2\ are members of \c\. \label{cases2}\ + txt \\G\<^sub>1\ is contained in \G\<^sub>2\ or vice versa, since both \G\<^sub>1\ and \G\<^sub>2\ + are members of \c\. \label{cases2}\ from cM G1 G2 consider "G1 \ G2" | "G2 \ G1" by (blast dest: chainsD) @@ -208,12 +205,11 @@ text \ \<^medskip> - The limit function \h\ is linear. Every element - \x\ in the domain of \h\ is in the domain of a function - \h'\ in the chain of norm preserving extensions. Furthermore, - \h\ is an extension of \h'\ so the function values of - \x\ are identical for \h'\ and \h\. Finally, the - function \h'\ is linear by construction of \M\. + The limit function \h\ is linear. Every element \x\ in the domain of \h\ + is in the domain of a function \h'\ in the chain of norm preserving + extensions. Furthermore, \h\ is an extension of \h'\ so the function + values of \x\ are identical for \h'\ and \h\. Finally, the function \h'\ + is linear by construction of \M\. \ lemma sup_lf: @@ -264,10 +260,9 @@ text \ \<^medskip> - The limit of a non-empty chain of norm preserving - extensions of \f\ is an extension of \f\, since every - element of the chain is an extension of \f\ and the supremum - is an extension for every element of the chain. + The limit of a non-empty chain of norm preserving extensions of \f\ is an + extension of \f\, since every element of the chain is an extension of \f\ + and the supremum is an extension for every element of the chain. \ lemma sup_ext: @@ -291,9 +286,8 @@ text \ \<^medskip> - The domain \H\ of the limit function is a superspace - of \F\, since \F\ is a subset of \H\. The - existence of the \0\ element in \F\ and the closure + The domain \H\ of the limit function is a superspace of \F\, since \F\ is + a subset of \H\. The existence of the \0\ element in \F\ and the closure properties follow from the fact that \F\ is a vector space. \ @@ -317,8 +311,7 @@ text \ \<^medskip> - The domain \H\ of the limit function is a subspace of - \E\. + The domain \H\ of the limit function is a subspace of \E\. \ lemma sup_subE: @@ -374,8 +367,8 @@ text \ \<^medskip> - The limit function is bounded by the norm \p\ as - well, since all elements in the chain are bounded by \p\. + The limit function is bounded by the norm \p\ as well, since all elements + in the chain are bounded by \p\. \ lemma sup_norm_pres: @@ -396,10 +389,10 @@ text \ \<^medskip> - The following lemma is a property of linear forms on real - vector spaces. It will be used for the lemma \abs_Hahn_Banach\ - (see page \pageref{abs-Hahn_Banach}). \label{abs-ineq-iff} For real - vector spaces the following inequations are equivalent: + The following lemma is a property of linear forms on real vector spaces. + It will be used for the lemma \abs_Hahn_Banach\ (see page + \pageref{abs-Hahn-Banach}). \label{abs-ineq-iff} For real vector spaces + the following inequality are equivalent: \begin{center} \begin{tabular}{lll} \\x \ H. \h x\ \ p x\ & and & diff -r a29295dac1ca -r f92bf6674699 src/HOL/Hahn_Banach/Linearform.thy --- a/src/HOL/Hahn_Banach/Linearform.thy Mon Nov 02 11:10:28 2015 +0100 +++ b/src/HOL/Hahn_Banach/Linearform.thy Mon Nov 02 11:43:02 2015 +0100 @@ -9,8 +9,8 @@ begin text \ - A \<^emph>\linear form\ is a function on a vector space into the reals - that is additive and multiplicative. + A \<^emph>\linear form\ is a function on a vector space into the reals that is + additive and multiplicative. \ locale linearform = diff -r a29295dac1ca -r f92bf6674699 src/HOL/Hahn_Banach/Normed_Space.thy --- a/src/HOL/Hahn_Banach/Normed_Space.thy Mon Nov 02 11:10:28 2015 +0100 +++ b/src/HOL/Hahn_Banach/Normed_Space.thy Mon Nov 02 11:43:02 2015 +0100 @@ -11,9 +11,9 @@ subsection \Quasinorms\ text \ - A \<^emph>\seminorm\ \\\\\ is a function on a real vector space - into the reals that has the following properties: it is positive - definite, absolute homogeneous and subadditive. + A \<^emph>\seminorm\ \\\\\ is a function on a real vector space into the reals + that has the following properties: it is positive definite, absolute + homogeneous and subadditive. \ locale seminorm = diff -r a29295dac1ca -r f92bf6674699 src/HOL/Hahn_Banach/Subspace.thy --- a/src/HOL/Hahn_Banach/Subspace.thy Mon Nov 02 11:10:28 2015 +0100 +++ b/src/HOL/Hahn_Banach/Subspace.thy Mon Nov 02 11:43:02 2015 +0100 @@ -11,9 +11,8 @@ subsection \Definition\ text \ - A non-empty subset \U\ of a vector space \V\ is a - \<^emph>\subspace\ of \V\, iff \U\ is closed under addition - and scalar multiplication. + A non-empty subset \U\ of a vector space \V\ is a \<^emph>\subspace\ of \V\, iff + \U\ is closed under addition and scalar multiplication. \ locale subspace = @@ -51,9 +50,9 @@ text \ \<^medskip> - Similar as for linear spaces, the existence of the zero - element in every subspace follows from the non-emptiness of the - carrier set and by vector space laws. + Similar as for linear spaces, the existence of the zero element in every + subspace follows from the non-emptiness of the carrier set and by vector + space laws. \ lemma (in subspace) zero [intro]: @@ -140,8 +139,8 @@ subsection \Linear closure\ text \ - The \<^emph>\linear closure\ of a vector \x\ is the set of all - scalar multiples of \x\. + The \<^emph>\linear closure\ of a vector \x\ is the set of all scalar multiples + of \x\. \ definition lin :: "('a::{minus,plus,zero}) \ 'a set" @@ -227,8 +226,8 @@ subsection \Sum of two vectorspaces\ text \ - The \<^emph>\sum\ of two vectorspaces \U\ and \V\ is the - set of all sums of elements from \U\ and \V\. + The \<^emph>\sum\ of two vectorspaces \U\ and \V\ is the set of all sums of + elements from \U\ and \V\. \ lemma sum_def: "U + V = {u + v | u v. u \ U \ v \ V}" @@ -329,10 +328,10 @@ subsection \Direct sums\ text \ - The sum of \U\ and \V\ is called \<^emph>\direct\, iff the - zero element is the only common element of \U\ and \V\. For every element \x\ of the direct sum of \U\ and - \V\ the decomposition in \x = u + v\ with - \u \ U\ and \v \ V\ is unique. + The sum of \U\ and \V\ is called \<^emph>\direct\, iff the zero element is the + only common element of \U\ and \V\. For every element \x\ of the direct + sum of \U\ and \V\ the decomposition in \x = u + v\ with \u \ U\ and + \v \ V\ is unique. \ lemma decomp: @@ -377,12 +376,10 @@ qed text \ - An application of the previous lemma will be used in the proof of - the Hahn-Banach Theorem (see page \pageref{decomp-H-use}): for any - element \y + a \ x\<^sub>0\ of the direct sum of a - vectorspace \H\ and the linear closure of \x\<^sub>0\ - the components \y \ H\ and \a\ are uniquely - determined. + An application of the previous lemma will be used in the proof of the + Hahn-Banach Theorem (see page \pageref{decomp-H-use}): for any element + \y + a \ x\<^sub>0\ of the direct sum of a vectorspace \H\ and the linear closure + of \x\<^sub>0\ the components \y \ H\ and \a\ are uniquely determined. \ lemma decomp_H': @@ -436,10 +433,9 @@ qed text \ - Since for any element \y + a \ x'\ of the direct sum of a - vectorspace \H\ and the linear closure of \x'\ the - components \y \ H\ and \a\ are unique, it follows from - \y \ H\ that \a = 0\. + Since for any element \y + a \ x'\ of the direct sum of a vectorspace \H\ + and the linear closure of \x'\ the components \y \ H\ and \a\ are unique, + it follows from \y \ H\ that \a = 0\. \ lemma decomp_H'_H: @@ -464,9 +460,8 @@ qed text \ - The components \y \ H\ and \a\ in \y + a \ x'\ - are unique, so the function \h'\ defined by - \h' (y + a \ x') = h y + a \ \\ is definite. + The components \y \ H\ and \a\ in \y + a \ x'\ are unique, so the function + \h'\ defined by \h' (y + a \ x') = h y + a \ \\ is definite. \ lemma h'_definite: diff -r a29295dac1ca -r f92bf6674699 src/HOL/Hahn_Banach/Vector_Space.thy --- a/src/HOL/Hahn_Banach/Vector_Space.thy Mon Nov 02 11:10:28 2015 +0100 +++ b/src/HOL/Hahn_Banach/Vector_Space.thy Mon Nov 02 11:43:02 2015 +0100 @@ -11,9 +11,9 @@ subsection \Signature\ text \ - For the definition of real vector spaces a type @{typ 'a} of the - sort \{plus, minus, zero}\ is considered, on which a real - scalar multiplication \\\ is declared. + For the definition of real vector spaces a type @{typ 'a} of the sort + \{plus, minus, zero}\ is considered, on which a real scalar multiplication + \\\ is declared. \ consts @@ -23,13 +23,13 @@ subsection \Vector space laws\ text \ - A \<^emph>\vector space\ is a non-empty set \V\ of elements from - @{typ 'a} with the following vector space laws: The set \V\ is - closed under addition and scalar multiplication, addition is - associative and commutative; \- x\ is the inverse of \x\ w.~r.~t.~addition and \0\ is the neutral element of - addition. Addition and multiplication are distributive; scalar - multiplication is associative and the real number \1\ is - the neutral element of scalar multiplication. + A \<^emph>\vector space\ is a non-empty set \V\ of elements from @{typ 'a} with + the following vector space laws: The set \V\ is closed under addition and + scalar multiplication, addition is associative and commutative; \- x\ is + the inverse of \x\ wrt.\ addition and \0\ is the neutral element of + addition. Addition and multiplication are distributive; scalar + multiplication is associative and the real number \1\ is the neutral + element of scalar multiplication. \ locale vectorspace = @@ -64,7 +64,8 @@ lemma neg_closed [iff]: "x \ V \ - x \ V" by (simp add: negate_eq1) -lemma add_left_commute: "x \ V \ y \ V \ z \ V \ x + (y + z) = y + (x + z)" +lemma add_left_commute: + "x \ V \ y \ V \ z \ V \ x + (y + z) = y + (x + z)" proof - assume xyz: "x \ V" "y \ V" "z \ V" then have "x + (y + z) = (x + y) + z" @@ -77,8 +78,8 @@ lemmas add_ac = add_assoc add_commute add_left_commute -text \The existence of the zero element of a vector space - follows from the non-emptiness of carrier set.\ +text \The existence of the zero element of a vector space follows from the + non-emptiness of carrier set.\ lemma zero [iff]: "0 \ V" proof - @@ -213,7 +214,8 @@ then show "x + y = x + z" by (simp only:) qed -lemma add_right_cancel: "x \ V \ y \ V \ z \ V \ (y + x = z + x) = (y = z)" +lemma add_right_cancel: + "x \ V \ y \ V \ z \ V \ (y + x = z + x) = (y = z)" by (simp only: add_commute add_left_cancel) lemma add_assoc_cong: @@ -371,4 +373,3 @@ end end - diff -r a29295dac1ca -r f92bf6674699 src/HOL/Hahn_Banach/document/root.tex --- a/src/HOL/Hahn_Banach/document/root.tex Mon Nov 02 11:10:28 2015 +0100 +++ b/src/HOL/Hahn_Banach/document/root.tex Mon Nov 02 11:43:02 2015 +0100 @@ -16,7 +16,7 @@ \pagenumbering{arabic} \title{The Hahn-Banach Theorem \\ for Real Vector Spaces} -\author{Gertrud Bauer \\ \url{http://www.in.tum.de/~bauerg/}} +\author{Gertrud Bauer} \maketitle \begin{abstract}