src/HOL/Hahn_Banach/Hahn_Banach_Sup_Lemmas.thy
changeset 60412 285c7ff27728
parent 58889 5b7a9633cfa8
child 60458 0d10ae17e3ee
equal deleted inserted replaced
60411:8f7e1279251d 60412:285c7ff27728
   418   next
   418   next
   419     assume r: ?R
   419     assume r: ?R
   420     show ?L
   420     show ?L
   421     proof
   421     proof
   422       fix x assume x: "x \<in> H"
   422       fix x assume x: "x \<in> H"
   423       show "\<And>a b :: real. - a \<le> b \<Longrightarrow> b \<le> a \<Longrightarrow> \<bar>b\<bar> \<le> a"
   423       show "- a \<le> b \<Longrightarrow> b \<le> a \<Longrightarrow> \<bar>b\<bar> \<le> a" for a b :: real
   424         by arith
   424         by arith
   425       from \<open>linearform H h\<close> and H x
   425       from \<open>linearform H h\<close> and H x
   426       have "- h x = h (- x)" by (rule linearform.neg [symmetric])
   426       have "- h x = h (- x)" by (rule linearform.neg [symmetric])
   427       also
   427       also
   428       from H x have "- x \<in> H" by (rule vectorspace.neg_closed)
   428       from H x have "- x \<in> H" by (rule vectorspace.neg_closed)