src/HOL/Multivariate_Analysis/Convex_Euclidean_Space.thy
changeset 61762 d50b993b4fb9
parent 61738 c4f6031f1310
child 61808 fc1556774cfe
equal deleted inserted replaced
61757:0d399131008f 61762:d50b993b4fb9
  4395     apply rule
  4395     apply rule
  4396     apply (rule ccontr)
  4396     apply (rule ccontr)
  4397     using \<open>y \<in> s\<close>
  4397     using \<open>y \<in> s\<close>
  4398   proof -
  4398   proof -
  4399     show "inner (y - z) z < inner (y - z) y"
  4399     show "inner (y - z) z < inner (y - z) y"
  4400       apply (subst diff_less_iff(1)[symmetric])
  4400       apply (subst diff_gt_0_iff_gt [symmetric])
  4401       unfolding inner_diff_right[symmetric] and inner_gt_zero_iff
  4401       unfolding inner_diff_right[symmetric] and inner_gt_zero_iff
  4402       using \<open>y\<in>s\<close> \<open>z\<notin>s\<close>
  4402       using \<open>y\<in>s\<close> \<open>z\<notin>s\<close>
  4403       apply auto
  4403       apply auto
  4404       done
  4404       done
  4405   next
  4405   next