src/HOL/Real_Vector_Spaces.thy
changeset 68532 f8b98d31ad45
parent 68499 d4312962161a
child 68594 5b05ede597b8
equal deleted inserted replaced
68528:d31e986fbebc 68532:f8b98d31ad45
  1090   then have "dist x1 x4 < (e/3 + e/3) + e/3"
  1090   then have "dist x1 x4 < (e/3 + e/3) + e/3"
  1091     by (metis assms(3) dist_commute dist_triangle_less_add)
  1091     by (metis assms(3) dist_commute dist_triangle_less_add)
  1092   then show ?thesis
  1092   then show ?thesis
  1093     by simp
  1093     by simp
  1094 qed
  1094 qed
  1095 
  1095   
  1096 subclass uniform_space
  1096 subclass uniform_space
  1097 proof
  1097 proof
  1098   fix E x
  1098   fix E x
  1099   assume "eventually E uniformity"
  1099   assume "eventually E uniformity"
  1100   then obtain e where E: "0 < e" "\<And>x y. dist x y < e \<Longrightarrow> E (x, y)"
  1100   then obtain e where E: "0 < e" "\<And>x y. dist x y < e \<Longrightarrow> E (x, y)"