src/HOL/Real_Vector_Spaces.thy
changeset 62087 44841d07ef1d
parent 62049 b0f941e207cf
child 62101 26c0a70f78a3
--- a/src/HOL/Real_Vector_Spaces.thy	Wed Jan 06 16:17:50 2016 +0100
+++ b/src/HOL/Real_Vector_Spaces.thy	Thu Jan 07 17:40:55 2016 +0000
@@ -1056,6 +1056,8 @@
   shows "x \<noteq> y \<longleftrightarrow> 0 < dist x y"
 by (simp add: zero_less_dist_iff)
 
+declare dist_nz [symmetric, simp]
+
 lemma dist_triangle_le:
   shows "dist x z + dist y z <= e \<Longrightarrow> dist x y <= e"
 by (rule order_trans [OF dist_triangle2])
@@ -1673,7 +1675,7 @@
 lemma eventually_at:
   fixes a :: "'a :: metric_space"
   shows "eventually P (at a within S) \<longleftrightarrow> (\<exists>d>0. \<forall>x\<in>S. x \<noteq> a \<and> dist x a < d \<longrightarrow> P x)"
-  unfolding eventually_at_filter eventually_nhds_metric by (auto simp: dist_nz)
+  unfolding eventually_at_filter eventually_nhds_metric by auto
 
 lemma eventually_at_le:
   fixes a :: "'a::metric_space"