changeset 51002 | 496013a6eb38 |
parent 49962 | a8cc904a6820 |
child 51478 | 270b21f3ae0a |
--- a/src/HOL/Library/Product_Vector.thy Thu Jan 31 12:09:07 2013 +0100 +++ b/src/HOL/Library/Product_Vector.thy Thu Jan 31 17:42:12 2013 +0100 @@ -408,8 +408,6 @@ instance proof fix r :: real and x y :: "'a \<times> 'b" - show "0 \<le> norm x" - unfolding norm_prod_def by simp show "norm x = 0 \<longleftrightarrow> x = 0" unfolding norm_prod_def by (simp add: prod_eq_iff)