src/HOL/Multivariate_Analysis/Euclidean_Space.thy
changeset 36586 4fa71a69d5b2
parent 36585 f2faab7b46e7
child 36587 534418d8d494
equal deleted inserted replaced
36585:f2faab7b46e7 36586:4fa71a69d5b2
   698   using sqrt_divide_self_eq[of x]
   698   using sqrt_divide_self_eq[of x]
   699   apply (simp add: inverse_eq_divide field_simps)
   699   apply (simp add: inverse_eq_divide field_simps)
   700   done
   700   done
   701 
   701 
   702 text{* Hence derive more interesting properties of the norm. *}
   702 text{* Hence derive more interesting properties of the norm. *}
   703 
       
   704 text {*
       
   705   This type-specific version is only here
       
   706   to make @{text normarith.ML} happy.
       
   707 *}
       
   708 lemma norm_0: "norm (0::real ^ _) = 0"
       
   709   by (rule norm_zero)
       
   710 
   703 
   711 lemma norm_mul[simp]: "norm(a *s x) = abs(a) * norm x"
   704 lemma norm_mul[simp]: "norm(a *s x) = abs(a) * norm x"
   712   by (simp add: norm_vector_def setL2_right_distrib abs_mult)
   705   by (simp add: norm_vector_def setL2_right_distrib abs_mult)
   713 
   706 
   714 lemma norm_eq_0_dot: "(norm x = 0) \<longleftrightarrow> (inner x x = (0::real))"
   707 lemma norm_eq_0_dot: "(norm x = 0) \<longleftrightarrow> (inner x x = (0::real))"