src/HOL/Analysis/Topology_Euclidean_Space.thy
changeset 68072 493b818e8e10
parent 67984 adc1a992c470
child 68120 2f161c6910f7
--- a/src/HOL/Analysis/Topology_Euclidean_Space.thy	Wed Apr 18 21:12:50 2018 +0100
+++ b/src/HOL/Analysis/Topology_Euclidean_Space.thy	Wed May 02 13:49:38 2018 +0200
@@ -10,18 +10,12 @@
 imports
   "HOL-Library.Indicator_Function"
   "HOL-Library.Countable_Set"
-  "HOL-Library.FuncSet"
   Linear_Algebra
   Norm_Arith
 begin
 
 (* FIXME: move elsewhere *)
 
-lemma Times_eq_image_sum:
-  fixes S :: "'a :: comm_monoid_add set" and T :: "'b :: comm_monoid_add set"
-  shows "S \<times> T = {u + v |u v. u \<in> (\<lambda>x. (x, 0)) ` S \<and> v \<in> Pair 0 ` T}"
-  by force
-
 lemma halfspace_Int_eq:
      "{x. a \<bullet> x \<le> b} \<inter> {x. b \<le> a \<bullet> x} = {x. a \<bullet> x = b}"
      "{x. b \<le> a \<bullet> x} \<inter> {x. a \<bullet> x \<le> b} = {x. a \<bullet> x = b}"