src/HOL/Analysis/Topology_Euclidean_Space.thy
changeset 66466 aec5d9c88d69
parent 66453 cc19f7ca2ed6
child 66641 ff2e0115fea4
--- a/src/HOL/Analysis/Topology_Euclidean_Space.thy	Sun Aug 20 03:35:20 2017 +0200
+++ b/src/HOL/Analysis/Topology_Euclidean_Space.thy	Sun Aug 20 18:55:03 2017 +0200
@@ -1736,6 +1736,17 @@
     by force
 qed
 
+lemma subset_box_complex:
+   "cbox a b \<subseteq> cbox c d \<longleftrightarrow> 
+      (Re a \<le> Re b \<and> Im a \<le> Im b) \<longrightarrow> Re a \<ge> Re c \<and> Im a \<ge> Im c \<and> Re b \<le> Re d \<and> Im b \<le> Im d"
+   "cbox a b \<subseteq> box c d \<longleftrightarrow> 
+      (Re a \<le> Re b \<and> Im a \<le> Im b) \<longrightarrow> Re a > Re c \<and> Im a > Im c \<and> Re b < Re d \<and> Im b < Im d"
+   "box a b \<subseteq> cbox c d \<longleftrightarrow>
+      (Re a < Re b \<and> Im a < Im b) \<longrightarrow> Re a \<ge> Re c \<and> Im a \<ge> Im c \<and> Re b \<le> Re d \<and> Im b \<le> Im d"
+   "box a b \<subseteq> box c d \<longleftrightarrow> 
+      (Re a < Re b \<and> Im a < Im b) \<longrightarrow> Re a \<ge> Re c \<and> Im a \<ge> Im c \<and> Re b \<le> Re d \<and> Im b \<le> Im d"
+  by (subst subset_box; force simp: Basis_complex_def)+
+
 lemma Int_interval:
   fixes a :: "'a::euclidean_space"
   shows "cbox a b \<inter> cbox c d =