# HG changeset patch # User wenzelm # Date 1446459028 -3600 # Node ID a29295dac1ca8425b072bfd03bef59405d0d39c9 # Parent bf4969660913658153c4e17e530a2f69c02683c4 isabelle update_cartouches -t; diff -r bf4969660913 -r a29295dac1ca src/HOL/Hahn_Banach/Function_Norm.thy --- a/src/HOL/Hahn_Banach/Function_Norm.thy Mon Nov 02 10:38:42 2015 +0100 +++ b/src/HOL/Hahn_Banach/Function_Norm.thy Mon Nov 02 11:10:28 2015 +0100 @@ -11,10 +11,10 @@ subsection \Continuous linear forms\ text \ - A linear form @{text f} on a normed vector space @{text "(V, \\\)"} + A linear form \f\ on a normed vector space \(V, \\\)\ is \<^emph>\continuous\, iff it is bounded, i.e. \begin{center} - @{text "\c \ R. \x \ V. \f x\ \ c \ \x\"} + \\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 @@ -42,33 +42,33 @@ subsection \The norm of a linear form\ text \ - The least real number @{text c} for which holds + The least real number \c\ for which holds \begin{center} - @{text "\x \ V. \f x\ \ c \ \x\"} + \\x \ V. \f x\ \ c \ \x\\ \end{center} - is called the \<^emph>\norm\ of @{text f}. + is called the \<^emph>\norm\ of \f\. - For non-trivial vector spaces @{text "V \ {0}"} the norm can be + For non-trivial vector spaces \V \ {0}\ the norm can be defined as \begin{center} - @{text "\f\ = \x \ 0. \f x\ / \x\"} + \\f\ = \x \ 0. \f x\ / \x\\ \end{center} - For the case @{text "V = {0}"} the supremum would be taken from an - empty set. Since @{text \} is unbounded, there would be no supremum. + 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 @{text "{} \ 0"} so that - @{text fn_norm} has the norm properties. Furthermore it does not - have to change the norm in all other cases, so it must be @{text 0}, - as all other elements are @{text "{} \ 0"}. + 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 @{text B} where the supremum is taken from as + Thus we define the set \B\ where the supremum is taken from as follows: \begin{center} - @{text "{0} \ {\f x\ / \x\. x \ 0 \ x \ F}"} + \{0} \ {\f x\ / \x\. x \ 0 \ x \ F}\ \end{center} - @{text fn_norm} is equal to the supremum of @{text B}, if the + \fn_norm\ is equal to the supremum of \B\, if the supremum exists (otherwise it is undefined). \ @@ -85,7 +85,7 @@ text \ The following lemma states that every continuous linear form on a - normed space @{text "(V, \\\)"} has a function norm. + normed space \(V, \\\)\ has a function norm. \ lemma (in normed_vectorspace_with_fn_norm) fn_norm_works: @@ -98,19 +98,19 @@ non-empty bounded set of reals has a supremum.\ have "\a. lub (B V f) a" proof (rule real_complete) - txt \First we have to show that @{text B} is non-empty:\ + txt \First we have to show that \B\ is non-empty:\ have "0 \ B V f" .. then show "\x. x \ B V f" .. - txt \Then we have to show that @{text B} is bounded:\ + txt \Then we have to show that \B\ is bounded:\ show "\c. \y \ B V f. y \ c" proof - - txt \We know that @{text f} is bounded by some value @{text c}.\ + 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 - @{text b}, such that @{text "y \ b"} for all @{text "y \ - B"}. Due to the definition of @{text B} there are two cases.\ + \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" @@ -121,8 +121,8 @@ assume "y = 0" then show ?thesis unfolding b_def by arith next - txt \The second case is @{text "y = \f x\ / \x\"} for some - @{text "x \ V"} with @{text "x \ 0"}.\ + txt \The second case is \y = \f x\ / \x\\ for some + \x \ V\ with \x \ 0\.\ assume "y \ 0" with y obtain x where y_rep: "y = \f x\ * inverse \x\" and x: "x \ V" and neq: "x \ 0" @@ -130,7 +130,7 @@ from x neq have gt: "0 < \x\" .. txt \The thesis follows by a short calculation using the - fact that @{text f} is bounded.\ + fact that \f\ is bounded.\ note y_rep also have "\f x\ * inverse \x\ \ (c * \x\) * inverse \x\" @@ -177,16 +177,16 @@ from this and b show ?thesis .. qed -text \The norm of a continuous function is always @{text "\ 0"}.\ +text \The norm of a continuous function is always \\ 0\.\ lemma (in normed_vectorspace_with_fn_norm) fn_norm_ge_zero [iff]: assumes "continuous V f norm" shows "0 \ \f\\V" proof - interpret continuous V f norm by fact - txt \The function norm is defined as the supremum of @{text B}. - So it is @{text "\ 0"} if all elements in @{text B} are @{text "\ - 0"}, provided the supremum exists and @{text B} is not empty.\ + txt \The function norm is defined as the supremum of \B\. + So it is \\ 0\ if all elements in \B\ are \\ + 0\, provided the supremum exists and \B\ is not empty.\ have "lub (B V f) (\f\\V)" using \continuous V f norm\ by (rule fn_norm_works) moreover have "0 \ B V f" .. @@ -197,7 +197,7 @@ \<^medskip> The fundamental property of function norms is: \begin{center} - @{text "\f x\ \ \f\ \ \x\"} + \\f x\ \ \f\ \ \x\\ \end{center} \ @@ -240,7 +240,7 @@ The function norm is the least positive real number for which the following inequation holds: \begin{center} - @{text "\f x\ \ c \ \x\"} + \\f x\ \ c \ \x\\ \end{center} \ diff -r bf4969660913 -r a29295dac1ca src/HOL/Hahn_Banach/Function_Order.thy --- a/src/HOL/Hahn_Banach/Function_Order.thy Mon Nov 02 10:38:42 2015 +0100 +++ b/src/HOL/Hahn_Banach/Function_Order.thy Mon Nov 02 11:10:28 2015 +0100 @@ -11,10 +11,10 @@ subsection \The graph of a function\ text \ - We define the \<^emph>\graph\ of a (real) function @{text f} with - domain @{text F} as the set + We define the \<^emph>\graph\ of a (real) function \f\ with + domain \F\ as the set \begin{center} - @{text "{(x, f x). x \ F}"} + \{(x, f x). x \ F}\ \end{center} So we are modeling partial functions by specifying the domain and the mapping function. We use the term ``function'' also for its @@ -41,8 +41,8 @@ subsection \Functions ordered by domain extension\ text \ - A function @{text h'} is an extension of @{text h}, iff the graph of - @{text h} is a subset of the graph of @{text h'}. + A function \h'\ is an extension of \h\, iff the graph of + \h\ is a subset of the graph of \h'\. \ lemma graph_extI: @@ -60,8 +60,7 @@ subsection \Domain and function of a graph\ text \ - The inverse functions to @{text graph} are @{text domain} and @{text - funct}. + The inverse functions to \graph\ are \domain\ and \funct\. \ definition domain :: "'a graph \ 'a set" @@ -71,8 +70,8 @@ where "funct g = (\x. (SOME y. (x, y) \ g))" text \ - The following lemma states that @{text g} is the graph of a function - if the relation induced by @{text 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: @@ -94,10 +93,9 @@ subsection \Norm-preserving extensions of a function\ text \ - Given a linear form @{text f} on the space @{text F} and a seminorm - @{text p} on @{text E}. The set of all linear extensions of @{text - f}, to superspaces @{text H} of @{text F}, which are bounded by - @{text 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 bf4969660913 -r a29295dac1ca src/HOL/Hahn_Banach/Hahn_Banach.thy --- a/src/HOL/Hahn_Banach/Hahn_Banach.thy Mon Nov 02 10:38:42 2015 +0100 +++ b/src/HOL/Hahn_Banach/Hahn_Banach.thy Mon Nov 02 11:10:28 2015 +0100 @@ -17,34 +17,31 @@ paragraph \Hahn-Banach Theorem.\ text \ - Let @{text F} be a subspace of a real vector space @{text E}, let @{text - p} be a semi-norm on @{text E}, and @{text f} be a linear form defined on - @{text F} such that @{text f} is bounded by @{text p}, i.e. @{text "\x \ - F. f x \ p x"}. Then @{text f} can be extended to a linear form @{text h} - on @{text E} such that @{text h} is norm-preserving, i.e. @{text h} is - also bounded by @{text 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 @{text M} as the set of norm-preserving extensions of - @{text f} to subspaces of @{text E}. The linear forms in @{text M} + \<^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 @{text M} has an upper - bound in @{text 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 - @{text g} in @{text M}. + \g\ in \M\. - \<^enum> The domain @{text H} of @{text g} is the whole space @{text - E}, as shown by classical contradiction: + \<^enum> The domain \H\ of \g\ is the whole space \E\, as shown by classical contradiction: - \<^item> Assuming @{text g} is not defined on whole @{text E}, it can - still be extended in a norm-preserving way to a super-space @{text - H'} of @{text 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 @{text g} can not be maximal. Contradiction! + \<^item> Thus \g\ can not be maximal. Contradiction! \ theorem Hahn_Banach: @@ -52,9 +49,9 @@ and "seminorm E p" and "linearform F f" assumes fp: "\x \ F. f x \ p x" shows "\h. linearform E h \ (\x \ F. h x = f x) \ (\x \ E. h x \ p x)" - -- \Let @{text E} be a vector space, @{text F} a subspace of @{text E}, @{text p} a seminorm on @{text E},\ - -- \and @{text f} a linear form on @{text F} such that @{text f} is bounded by @{text p},\ - -- \then @{text f} can be extended to a linear form @{text h} on @{text E} in a norm-preserving way. \<^smallskip>\ + -- \Let \E\ be a vector space, \F\ a subspace of \E\, \p\ a seminorm on \E\,\ + -- \and \f\ a linear form on \F\ such that \f\ is bounded by \p\,\ + -- \then \f\ can be extended to a linear form \h\ on \E\ in a norm-preserving way. \<^smallskip>\ proof - interpret vectorspace E by fact interpret subspace F E by fact @@ -67,8 +64,8 @@ { fix c assume cM: "c \ chains M" and ex: "\x. x \ c" have "\c \ M" - -- \Show that every non-empty chain @{text c} of @{text M} has an upper bound in @{text M}:\ - -- \@{text "\c"} is greater than any element of the chain @{text c}, so it suffices to show @{text "\c \ M"}.\ + -- \Show that every non-empty chain \c\ of \M\ has an upper bound in \M\:\ + -- \\\c\ is greater than any element of the chain \c\, so it suffices to show \\c \ M\.\ unfolding M_def proof (rule norm_pres_extensionI) let ?H = "domain (\c)" @@ -98,9 +95,9 @@ qed } then have "\g \ M. \x \ M. g \ x \ x = g" - -- \With Zorn's Lemma we can conclude that there is a maximal element in @{text M}. \<^smallskip>\ + -- \With Zorn's Lemma we can conclude that there is a maximal element in \M\. \<^smallskip>\ proof (rule Zorn's_Lemma) - -- \We show that @{text M} is non-empty:\ + -- \We show that \M\ is non-empty:\ show "graph F f \ M" unfolding M_def proof (rule norm_pres_extensionI2) @@ -119,18 +116,18 @@ and HE: "H \ E" and FH: "F \ H" and graphs: "graph F f \ graph H h" and hp: "\x \ H. h x \ p x" unfolding M_def .. - -- \@{text g} is a norm-preserving extension of @{text f}, in other words:\ - -- \@{text g} is the graph of some linear form @{text h} defined on a subspace @{text H} of @{text E},\ - -- \and @{text h} is an extension of @{text f} that is again bounded by @{text p}. \<^smallskip>\ + -- \\g\ is a norm-preserving extension of \f\, in other words:\ + -- \\g\ is the graph of some linear form \h\ defined on a subspace \H\ of \E\,\ + -- \and \h\ is an extension of \f\ that is again bounded by \p\. \<^smallskip>\ from HE E have H: "vectorspace H" by (rule subspace.vectorspace) have HE_eq: "H = E" - -- \We show that @{text h} is defined on whole @{text E} by classical contradiction. \<^smallskip>\ + -- \We show that \h\ is defined on whole \E\ by classical contradiction. \<^smallskip>\ proof (rule classical) assume neq: "H \ E" - -- \Assume @{text h} is not defined on whole @{text E}. Then show that @{text h} can be extended\ - -- \in a norm-preserving way to a function @{text h'} with the graph @{text g'}. \<^smallskip>\ + -- \Assume \h\ is not defined on whole \E\. Then show that \h\ can be extended\ + -- \in a norm-preserving way to a function \h'\ with the graph \g'\. \<^smallskip>\ have "\g' \ M. g \ g' \ g \ g'" proof - from HE have "H \ E" .. @@ -146,7 +143,7 @@ qed def H' \ "H + lin x'" - -- \Define @{text H'} as the direct sum of @{text H} and the linear closure of @{text x'}. \<^smallskip>\ + -- \Define \H'\ as the direct sum of \H\ and the linear closure of \x'\. \<^smallskip>\ have HH': "H \ H'" proof (unfold H'_def) from x'E have "vectorspace (lin x')" .. @@ -156,8 +153,8 @@ obtain xi where xi: "\y \ H. - p (y + x') - h y \ xi \ xi \ p (y + x') - h y" - -- \Pick a real number @{text \} that fulfills certain inequations; this will\ - -- \be used to establish that @{text h'} is a norm-preserving extension of @{text h}. + -- \Pick a real number \\\ that fulfills certain inequations; this will\ + -- \be used to establish that \h'\ is a norm-preserving extension of \h\. \label{ex-xi-use}\<^smallskip>\ proof - from H have "\xi. \y \ H. - p (y + x') - h y \ xi @@ -185,10 +182,10 @@ def h' \ "\x. let (y, a) = SOME (y, a). x = y + a \ x' \ y \ H in h y + a * xi" - -- \Define the extension @{text h'} of @{text h} to @{text H'} using @{text \}. \<^smallskip>\ + -- \Define the extension \h'\ of \h\ to \H'\ using \\\. \<^smallskip>\ have "g \ graph H' h' \ g \ graph H' h'" - -- \@{text h'} is an extension of @{text h} \dots \<^smallskip>\ + -- \\h'\ is an extension of \h\ \dots \<^smallskip>\ proof show "g \ graph H' h'" proof - @@ -225,7 +222,7 @@ qed qed moreover have "graph H' h' \ M" - -- \and @{text h'} is norm-preserving. \<^smallskip>\ + -- \and \h'\ is norm-preserving. \<^smallskip>\ proof (unfold M_def) show "graph H' h' \ norm_pres_extensions E p F f" proof (rule norm_pres_extensionI2) @@ -273,7 +270,7 @@ ultimately show ?thesis .. qed then have "\ (\x \ M. g \ x \ g = x)" by simp - -- \So the graph @{text g} of @{text h} cannot be maximal. Contradiction! \<^smallskip>\ + -- \So the graph \g\ of \h\ cannot be maximal. Contradiction! \<^smallskip>\ with gx show "H = E" by contradiction qed @@ -296,13 +293,13 @@ text \ The following alternative formulation of the Hahn-Banach Theorem\label{abs-Hahn-Banach} uses the fact that for a real linear - form @{text f} and a seminorm @{text p} the following inequations + 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}).} \begin{center} \begin{tabular}{lll} - @{text "\x \ H. \h x\ \ p x"} & and & - @{text "\x \ H. h x \ p x"} \\ + \\x \ H. \h x\ \ p x\ & and & + \\x \ H. h x \ p x\ \\ \end{tabular} \end{center} \ @@ -339,9 +336,9 @@ subsection \The Hahn-Banach Theorem for normed spaces\ text \ - Every continuous linear form @{text f} on a subspace @{text F} of a - norm space @{text E}, can be extended to a continuous linear form - @{text g} on @{text E} such that @{text "\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: @@ -370,22 +367,22 @@ by (rule normed_vectorspace_with_fn_norm.fn_norm_ge_zero [OF normed_vectorspace_with_fn_norm.intro, OF F_norm \continuous F f norm\ , folded B_def fn_norm_def]) - txt \We define a function @{text p} on @{text E} as follows: - @{text "p x = \f\ \ \x\"}\ + txt \We define a function \p\ on \E\ as follows: + \p x = \f\ \ \x\\\ def p \ "\x. \f\\F * \x\" - txt \@{text p} is a seminorm on @{text E}:\ + txt \\p\ is a seminorm on \E\:\ have q: "seminorm E p" proof fix x y a assume x: "x \ E" and y: "y \ E" - txt \@{text p} is positive definite:\ + txt \\p\ is positive definite:\ have "0 \ \f\\F" by (rule ge_zero) moreover from x have "0 \ \x\" .. ultimately show "0 \ p x" by (simp add: p_def zero_le_mult_iff) - txt \@{text p} is absolutely homogeneous:\ + txt \\p\ is absolutely homogeneous:\ show "p (a \ x) = \a\ * p x" proof - @@ -396,7 +393,7 @@ finally show ?thesis . qed - txt \Furthermore, @{text p} is subadditive:\ + txt \Furthermore, \p\ is subadditive:\ show "p (x + y) \ p x + p y" proof - @@ -411,7 +408,7 @@ qed qed - txt \@{text f} is bounded by @{text p}.\ + txt \\f\ is bounded by \p\.\ have "\x \ F. \f x\ \ p x" proof @@ -423,10 +420,10 @@ OF F_norm, folded B_def fn_norm_def]) qed - txt \Using the fact that @{text p} is a seminorm and @{text f} is bounded - by @{text p} we can apply the Hahn-Banach Theorem for real vector - spaces. So @{text f} can be extended in a norm-preserving way to - some function @{text g} on the whole vector space @{text 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" @@ -434,7 +431,7 @@ and b: "\x \ E. \g x\ \ p x" by (rule abs_Hahn_Banach [elim_format]) iprover - txt \We furthermore have to show that @{text g} is also continuous:\ + txt \We furthermore have to show that \g\ is also continuous:\ have g_cont: "continuous E g norm" using linearformE proof @@ -443,22 +440,21 @@ by (simp only: p_def) qed - txt \To complete the proof, we show that @{text "\g\ = \f\"}.\ + txt \To complete the proof, we show that \\g\ = \f\\.\ have "\g\\E = \f\\F" proof (rule order_antisym) txt \ - First we show @{text "\g\ \ \f\"}. The function norm @{text - "\g\"} is defined as the smallest @{text "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} - @{text "\x \ E. \g x\ \ c \ \x\"} + \\x \ E. \g x\ \ c \ \x\\ \end{tabular} \end{center} \noindent Furthermore holds \begin{center} \begin{tabular}{l} - @{text "\x \ E. \g x\ \ \f\ \ \x\"} + \\x \ E. \g x\ \ \f\ \ \x\\ \end{tabular} \end{center} \ diff -r bf4969660913 -r a29295dac1ca src/HOL/Hahn_Banach/Hahn_Banach_Ext_Lemmas.thy --- a/src/HOL/Hahn_Banach/Hahn_Banach_Ext_Lemmas.thy Mon Nov 02 10:38:42 2015 +0100 +++ b/src/HOL/Hahn_Banach/Hahn_Banach_Ext_Lemmas.thy Mon Nov 02 11:10:28 2015 +0100 @@ -9,34 +9,32 @@ begin text \ - In this section the following context is presumed. Let @{text E} be - a real vector space with a seminorm @{text q} on @{text E}. @{text - F} is a subspace of @{text E} and @{text f} a linear function on - @{text F}. We consider a subspace @{text H} of @{text E} that is a - superspace of @{text F} and a linear form @{text h} on @{text - H}. @{text H} is a not equal to @{text E} and @{text "x\<^sub>0"} is - an element in @{text "E - H"}. @{text H} is extended to the direct - sum @{text "H' = H + lin x\<^sub>0"}, so for any @{text "x \ H'"} - the decomposition of @{text "x = y + a \ x"} with @{text "y \ H"} is - unique. @{text h'} is defined on @{text H'} by @{text "h' x = h y + - a \ \"} for a certain @{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 \\\. - Subsequently we show some properties of this extension @{text h'} of - @{text 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 @{text f} (see page \pageref{ex-xi-use}). It is a - consequence of the completeness of @{text \}. To show + extension of \f\ (see page \pageref{ex-xi-use}). It is a + consequence of the completeness of \\\. To show \begin{center} \begin{tabular}{l} - @{text "\\. \y \ F. a y \ \ \ \ \ b y"} + \\\. \y \ F. a y \ \ \ \ \ b y\ \end{tabular} \end{center} \noindent it suffices to show that \begin{center} \begin{tabular}{l} - @{text "\u \ F. \v \ F. a u \ b v"} + \\u \ F. \v \ F. a u \ b v\ \end{tabular} \end{center} \ @@ -48,7 +46,7 @@ proof - interpret vectorspace F by fact txt \From the completeness of the reals follows: - The set @{text "S = {a u. u \ F}"} has a supremum, if it is + The set \S = {a u. u \ F}\ has a supremum, if it is non-empty and has an upper bound.\ let ?S = "{a u | u. u \ F}" @@ -86,9 +84,9 @@ text \ \<^medskip> - The function @{text h'} is defined as a @{text "h' x = h y - + a \ \"} where @{text "x = y + a \ \"} is a linear extension of - @{text h} to @{text 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: @@ -194,8 +192,8 @@ text \ \<^medskip> - The linear extension @{text h'} of @{text h} - is bounded by the seminorm @{text 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) = @@ -235,8 +233,8 @@ also from x0 y' z have "p y = p (y + a \ x0)" by simp finally show ?thesis . next - txt \In the case @{text "a < 0"}, we use @{text "a\<^sub>1"} - with @{text ya} taken as @{text "y / a"}:\ + txt \In the case \a < 0\, we use \a\<^sub>1\ + with \ya\ taken as \y / a\:\ assume lz: "a < 0" then have nz: "a \ 0" by simp from a1 ay have "- p (inverse a \ y + x0) - h (inverse a \ y) \ xi" .. @@ -257,8 +255,8 @@ finally have "a * xi \ p (y + a \ x0) - h y" . then show ?thesis by simp next - txt \In the case @{text "a > 0"}, we use @{text "a\<^sub>2"} - with @{text ya} taken as @{text "y / a"}:\ + txt \In the case \a > 0\, we use \a\<^sub>2\ + with \ya\ taken as \y / a\:\ assume gz: "0 < a" then have nz: "a \ 0" by simp from a2 ay have "xi \ p (inverse a \ y + x0) - h (inverse a \ y)" .. diff -r bf4969660913 -r a29295dac1ca src/HOL/Hahn_Banach/Hahn_Banach_Sup_Lemmas.thy --- a/src/HOL/Hahn_Banach/Hahn_Banach_Sup_Lemmas.thy Mon Nov 02 10:38:42 2015 +0100 +++ b/src/HOL/Hahn_Banach/Hahn_Banach_Sup_Lemmas.thy Mon Nov 02 11:10:28 2015 +0100 @@ -11,17 +11,17 @@ 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 @{text E} be a real vector space with a seminorm - @{text p} on @{text E}. @{text F} is a subspace of @{text E} and - @{text f} a linear form on @{text F}. We consider a chain @{text c} - of norm-preserving extensions of @{text f}, such that @{text "\c = - graph H h"}. We will show some properties about the limit function - @{text h}, i.e.\ the supremum of the chain @{text c}. + 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 @{text c} be a chain of norm-preserving extensions of - the function @{text f} and let @{text "graph H h"} be the supremum - of @{text c}. Every element in @{text H} is member of one of the + 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. \ @@ -57,11 +57,10 @@ text \ \<^medskip> - Let @{text c} be a chain of norm-preserving extensions of - the function @{text f} and let @{text "graph H h"} be the supremum - of @{text c}. Every element in the domain @{text H} of the supremum - function is member of the domain @{text H'} of some function @{text - h'}, such that @{text h} extends @{text 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': @@ -86,10 +85,10 @@ text \ \<^medskip> - Any two elements @{text x} and @{text y} in the domain - @{text H} of the supremum function @{text h} are both in the domain - @{text H'} of some function @{text h'}, such that @{text h} extends - @{text 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: @@ -103,8 +102,8 @@ \ linearform H' h' \ H' \ E \ F \ H' \ graph F f \ graph H' h' \ (\x \ H'. h' x \ p x)" proof - - txt \@{text y} is in the domain @{text H''} of some function @{text h''}, - such that @{text h} extends @{text h''}.\ + txt \\y\ is in the domain \H''\ of some function \h''\, + such that \h\ extends \h''\.\ from M cM u and y obtain H' h' where y_hy: "(y, h y) \ graph H' h'" @@ -114,8 +113,8 @@ "graph F f \ graph H' h'" "\x \ H'. h' x \ p x" by (rule some_H'h't [elim_format]) blast - txt \@{text x} is in the domain @{text H'} of some function @{text h'}, - such that @{text h} extends @{text h'}.\ + txt \\x\ is in the domain \H'\ of some function \h'\, + such that \h\ extends \h'\.\ from M cM u and x obtain H'' h'' where x_hx: "(x, h x) \ graph H'' h''" @@ -125,9 +124,9 @@ "graph F f \ graph H'' h''" "\x \ H''. h'' x \ p x" by (rule some_H'h't [elim_format]) blast - txt \Since both @{text h'} and @{text h''} are elements of the chain, - @{text h''} is an extension of @{text h'} or vice versa. Thus both - @{text x} and @{text y} are contained in the greater + txt \Since both \h'\ and \h''\ are elements of the chain, + \h''\ is an extension of \h'\ or vice versa. Thus both + \x\ and \y\ are contained in the greater one. \label{cases1}\ from cM c'' c' consider "graph H'' h'' \ graph H' h'" | "graph H' h' \ graph H'' h''" @@ -160,7 +159,7 @@ text \ \<^medskip> The relation induced by the graph of the supremum of a - chain @{text c} is definite, i.~e.~t is the graph of a function. + chain \c\ is definite, i.~e.~t is the graph of a function. \ lemma sup_definite: @@ -182,9 +181,8 @@ then obtain H2 h2 where G2_rep: "G2 = graph H2 h2" unfolding M_def by blast - txt \@{text "G\<^sub>1"} is contained in @{text "G\<^sub>2"} - or vice versa, since both @{text "G\<^sub>1"} and @{text - "G\<^sub>2"} are members of @{text 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) @@ -210,12 +208,12 @@ text \ \<^medskip> - The limit function @{text h} is linear. Every element - @{text x} in the domain of @{text h} is in the domain of a function - @{text h'} in the chain of norm preserving extensions. Furthermore, - @{text h} is an extension of @{text h'} so the function values of - @{text x} are identical for @{text h'} and @{text h}. Finally, the - function @{text h'} is linear by construction of @{text 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: @@ -267,8 +265,8 @@ text \ \<^medskip> The limit of a non-empty chain of norm preserving - extensions of @{text f} is an extension of @{text f}, since every - element of the chain is an extension of @{text f} and the supremum + 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. \ @@ -293,10 +291,10 @@ text \ \<^medskip> - The domain @{text H} of the limit function is a superspace - of @{text F}, since @{text F} is a subset of @{text H}. The - existence of the @{text 0} element in @{text F} and the closure - properties follow from the fact that @{text F} is a vector space. + 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. \ lemma sup_supF: @@ -319,8 +317,8 @@ text \ \<^medskip> - The domain @{text H} of the limit function is a subspace of - @{text E}. + The domain \H\ of the limit function is a subspace of + \E\. \ lemma sup_subE: @@ -376,8 +374,8 @@ text \ \<^medskip> - The limit function is bounded by the norm @{text p} as - well, since all elements in the chain are bounded by @{text 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: @@ -399,13 +397,13 @@ text \ \<^medskip> The following lemma is a property of linear forms on real - vector spaces. It will be used for the lemma @{text abs_Hahn_Banach} + 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: \begin{center} \begin{tabular}{lll} - @{text "\x \ H. \h x\ \ p x"} & and & - @{text "\x \ H. h x \ p x"} \\ + \\x \ H. \h x\ \ p x\ & and & + \\x \ H. h x \ p x\ \\ \end{tabular} \end{center} \ diff -r bf4969660913 -r a29295dac1ca src/HOL/Hahn_Banach/Linearform.thy --- a/src/HOL/Hahn_Banach/Linearform.thy Mon Nov 02 10:38:42 2015 +0100 +++ b/src/HOL/Hahn_Banach/Linearform.thy Mon Nov 02 11:10:28 2015 +0100 @@ -44,7 +44,7 @@ finally show ?thesis by simp qed -text \Every linear form yields @{text 0} for the @{text 0} vector.\ +text \Every linear form yields \0\ for the \0\ vector.\ lemma (in linearform) zero [iff]: assumes "vectorspace V" diff -r bf4969660913 -r a29295dac1ca src/HOL/Hahn_Banach/Normed_Space.thy --- a/src/HOL/Hahn_Banach/Normed_Space.thy Mon Nov 02 10:38:42 2015 +0100 +++ b/src/HOL/Hahn_Banach/Normed_Space.thy Mon Nov 02 11:10:28 2015 +0100 @@ -11,7 +11,7 @@ subsection \Quasinorms\ text \ - A \<^emph>\seminorm\ @{text "\\\"} is a function on a real vector space + 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. \ @@ -57,8 +57,8 @@ subsection \Norms\ text \ - A \<^emph>\norm\ @{text "\\\"} is a seminorm that maps only the - @{text 0} vector to @{text 0}. + A \<^emph>\norm\ \\\\\ is a seminorm that maps only the + \0\ vector to \0\. \ locale norm = seminorm + diff -r bf4969660913 -r a29295dac1ca src/HOL/Hahn_Banach/Subspace.thy --- a/src/HOL/Hahn_Banach/Subspace.thy Mon Nov 02 10:38:42 2015 +0100 +++ b/src/HOL/Hahn_Banach/Subspace.thy Mon Nov 02 11:10:28 2015 +0100 @@ -11,8 +11,8 @@ subsection \Definition\ text \ - A non-empty subset @{text U} of a vector space @{text V} is a - \<^emph>\subspace\ of @{text V}, iff @{text U} is closed under addition + 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. \ @@ -140,8 +140,8 @@ subsection \Linear closure\ text \ - The \<^emph>\linear closure\ of a vector @{text x} is the set of all - scalar multiples of @{text 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 +227,8 @@ subsection \Sum of two vectorspaces\ text \ - The \<^emph>\sum\ of two vectorspaces @{text U} and @{text V} is the - set of all sums of elements from @{text U} and @{text 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}" @@ -246,7 +246,7 @@ "u \ U \ v \ V \ u + v \ U + V" unfolding sum_def by blast -text \@{text U} is a subspace of @{text "U + V"}.\ +text \\U\ is a subspace of \U + V\.\ lemma subspace_sum1 [iff]: assumes "vectorspace U" "vectorspace V" @@ -329,11 +329,10 @@ subsection \Direct sums\ text \ - The sum of @{text U} and @{text V} is called \<^emph>\direct\, iff the - zero element is the only common element of @{text U} and @{text - V}. For every element @{text x} of the direct sum of @{text U} and - @{text V} the decomposition in @{text "x = u + v"} with - @{text "u \ U"} and @{text "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: @@ -380,9 +379,9 @@ 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 @{text "y + a \ x\<^sub>0"} of the direct sum of a - vectorspace @{text H} and the linear closure of @{text "x\<^sub>0"} - the components @{text "y \ H"} and @{text a} are uniquely + 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. \ @@ -437,10 +436,10 @@ qed text \ - Since for any element @{text "y + a \ x'"} of the direct sum of a - vectorspace @{text H} and the linear closure of @{text x'} the - components @{text "y \ H"} and @{text a} are unique, it follows from - @{text "y \ H"} that @{text "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: @@ -465,9 +464,9 @@ qed text \ - The components @{text "y \ H"} and @{text a} in @{text "y + a \ x'"} - are unique, so the function @{text h'} defined by - @{text "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 bf4969660913 -r a29295dac1ca src/HOL/Hahn_Banach/Vector_Space.thy --- a/src/HOL/Hahn_Banach/Vector_Space.thy Mon Nov 02 10:38:42 2015 +0100 +++ b/src/HOL/Hahn_Banach/Vector_Space.thy Mon Nov 02 11:10:28 2015 +0100 @@ -12,8 +12,8 @@ text \ For the definition of real vector spaces a type @{typ 'a} of the - sort @{text "{plus, minus, zero}"} is considered, on which a real - scalar multiplication @{text \} is declared. + sort \{plus, minus, zero}\ is considered, on which a real + scalar multiplication \\\ is declared. \ consts @@ -23,13 +23,12 @@ subsection \Vector space laws\ text \ - A \<^emph>\vector space\ is a non-empty set @{text V} of elements from - @{typ 'a} with the following vector space laws: The set @{text V} is + 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; @{text "- x"} is the inverse of @{text - x} w.~r.~t.~addition and @{text 0} is the neutral element of + 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 @{text "1"} is + multiplication is associative and the real number \1\ is the neutral element of scalar multiplication. \ diff -r bf4969660913 -r a29295dac1ca src/HOL/Hahn_Banach/Zorn_Lemma.thy --- a/src/HOL/Hahn_Banach/Zorn_Lemma.thy Mon Nov 02 10:38:42 2015 +0100 +++ b/src/HOL/Hahn_Banach/Zorn_Lemma.thy Mon Nov 02 11:10:28 2015 +0100 @@ -10,13 +10,12 @@ text \ Zorn's Lemmas states: if every linear ordered subset of an ordered - set @{text S} has an upper bound in @{text S}, then there exists a - maximal element in @{text S}. In our application, @{text S} is a + set \S\ has an upper bound in \S\, then there exists a + maximal element in \S\. In our application, \S\ is a set of sets ordered by set inclusion. Since the union of a chain of sets is an upper bound for all elements of the chain, the conditions - of Zorn's lemma can be modified: if @{text S} is non-empty, it - suffices to show that for every non-empty chain @{text c} in @{text - S} the union of @{text c} also lies in @{text S}. + of Zorn's lemma can be modified: if \S\ is non-empty, it + suffices to show that for every non-empty chain \c\ in \S\ the union of \c\ also lies in \S\. \ theorem Zorn's_Lemma: @@ -30,14 +29,14 @@ show "\y \ S. \z \ c. z \ y" proof cases - txt \If @{text c} is an empty chain, then every element in - @{text S} is an upper bound of @{text c}.\ + txt \If \c\ is an empty chain, then every element in + \S\ is an upper bound of \c\.\ assume "c = {}" with aS show ?thesis by fast - txt \If @{text c} is non-empty, then @{text "\c"} is an upper - bound of @{text c}, lying in @{text S}.\ + txt \If \c\ is non-empty, then \\c\ is an upper + bound of \c\, lying in \S\.\ next assume "c \ {}"