merged
authorpaulson
Sat, 02 Nov 2019 20:52:24 +0000
changeset 71005 7f1241a2bf30
parent 71003 699ff83813c0 (current diff)
parent 71004 b86d30707837 (diff)
child 71006 41685289b8eb
child 71008 e892f7a1fd83
merged
--- a/src/HOL/Analysis/Starlike.thy	Sat Nov 02 20:56:22 2019 +0100
+++ b/src/HOL/Analysis/Starlike.thy	Sat Nov 02 20:52:24 2019 +0000
@@ -3162,14 +3162,8 @@
     assume "z \<in> ?lhs"
     have *: "z = (fst z, snd z)"
       by auto
-    have "z \<in> ?rhs"
-      using rel_interior_convex_cone_aux[of S "fst z" "snd z"] assms \<open>z \<in> ?lhs\<close>
-      apply auto
-      apply (rule_tac x = "fst z" in exI)
-      apply (rule_tac x = x in exI)
-      using *
-      apply auto
-      done
+    then have "z \<in> ?rhs"
+      using rel_interior_convex_cone_aux[of S "fst z" "snd z"] assms \<open>z \<in> ?lhs\<close> by fastforce
   }
   moreover
   {