src/HOL/Lattices_Big.thy
changeset 63915 bab633745c7f
parent 63290 9ac558ab0906
child 65817 8ee1799fb076
--- a/src/HOL/Lattices_Big.thy	Sun Sep 18 17:59:28 2016 +0200
+++ b/src/HOL/Lattices_Big.thy	Sun Sep 18 20:33:48 2016 +0200
@@ -522,9 +522,11 @@
   assumes "finite A" and min: "\<And>b. b \<in> A \<Longrightarrow> a \<le> b"
   shows "Min (insert a A) = a"
 proof (cases "A = {}")
-  case True then show ?thesis by simp
+  case True
+  then show ?thesis by simp
 next
-  case False with \<open>finite A\<close> have "Min (insert a A) = min a (Min A)"
+  case False
+  with \<open>finite A\<close> have "Min (insert a A) = min a (Min A)"
     by simp
   moreover from \<open>finite A\<close> \<open>A \<noteq> {}\<close> min have "a \<le> Min A" by simp
   ultimately show ?thesis by (simp add: min.absorb1)
@@ -534,9 +536,11 @@
   assumes "finite A" and max: "\<And>b. b \<in> A \<Longrightarrow> b \<le> a"
   shows "Max (insert a A) = a"
 proof (cases "A = {}")
-  case True then show ?thesis by simp
+  case True
+  then show ?thesis by simp
 next
-  case False with \<open>finite A\<close> have "Max (insert a A) = max a (Max A)"
+  case False
+  with \<open>finite A\<close> have "Max (insert a A) = max a (Max A)"
     by simp
   moreover from \<open>finite A\<close> \<open>A \<noteq> {}\<close> max have "Max A \<le> a" by simp
   ultimately show ?thesis by (simp add: max.absorb1)