src/HOL/Set_Interval.thy
changeset 71699 8e5c20e4e11a
parent 71535 b612edee9b0c
child 71822 67cc2319104f
--- a/src/HOL/Set_Interval.thy	Mon Apr 06 11:56:04 2020 +0100
+++ b/src/HOL/Set_Interval.thy	Mon Apr 06 19:46:38 2020 +0100
@@ -812,10 +812,10 @@
     greaterThanLessThan_def)
 
 lemma atLeastAtMostSuc_conv: "m \<le> Suc n \<Longrightarrow> {m..Suc n} = insert (Suc n) {m..n}"
-by (auto simp add: atLeastAtMost_def)
+  by auto
 
 lemma atLeastAtMost_insertL: "m \<le> n \<Longrightarrow> insert m {Suc m..n} = {m ..n}"
-by auto
+  by auto
 
 text \<open>The analogous result is useful on \<^typ>\<open>int\<close>:\<close>
 (* here, because we don't have an own int section *)