src/HOL/Hahn_Banach/Hahn_Banach.thy
changeset 56749 e96d6b38649e
parent 52183 667961fa6a60
child 58622 aa99568f56de
equal deleted inserted replaced
56748:10b52ca3b4a2 56749:e96d6b38649e
   389     have "0 \<le> \<parallel>f\<parallel>\<hyphen>F" by (rule ge_zero)
   389     have "0 \<le> \<parallel>f\<parallel>\<hyphen>F" by (rule ge_zero)
   390     moreover from x have "0 \<le> \<parallel>x\<parallel>" ..
   390     moreover from x have "0 \<le> \<parallel>x\<parallel>" ..
   391     ultimately show "0 \<le> p x"  
   391     ultimately show "0 \<le> p x"  
   392       by (simp add: p_def zero_le_mult_iff)
   392       by (simp add: p_def zero_le_mult_iff)
   393 
   393 
   394     txt {* @{text p} is absolutely homogenous: *}
   394     txt {* @{text p} is absolutely homogeneous: *}
   395 
   395 
   396     show "p (a \<cdot> x) = \<bar>a\<bar> * p x"
   396     show "p (a \<cdot> x) = \<bar>a\<bar> * p x"
   397     proof -
   397     proof -
   398       have "p (a \<cdot> x) = \<parallel>f\<parallel>\<hyphen>F * \<parallel>a \<cdot> x\<parallel>" by (simp only: p_def)
   398       have "p (a \<cdot> x) = \<parallel>f\<parallel>\<hyphen>F * \<parallel>a \<cdot> x\<parallel>" by (simp only: p_def)
   399       also from x have "\<parallel>a \<cdot> x\<parallel> = \<bar>a\<bar> * \<parallel>x\<parallel>" by (rule abs_homogenous)
   399       also from x have "\<parallel>a \<cdot> x\<parallel> = \<bar>a\<bar> * \<parallel>x\<parallel>" by (rule abs_homogenous)