src/HOL/SetInterval.thy
changeset 17719 2e75155c5ed5
parent 17149 e2b19c92ef51
child 19022 0e6ec4fd204c
equal deleted inserted replaced
17718:9dab1e491d10 17719:2e75155c5ed5
   194   by (auto simp add: atLeastAtMost_def atMost_def atLeast_def);
   194   by (auto simp add: atLeastAtMost_def atMost_def atLeast_def);
   195 
   195 
   196 lemma atLeastLessThan_empty[simp]: "n \<le> m ==> {m..<n::'a::order} = {}"
   196 lemma atLeastLessThan_empty[simp]: "n \<le> m ==> {m..<n::'a::order} = {}"
   197 by (auto simp add: atLeastLessThan_def)
   197 by (auto simp add: atLeastLessThan_def)
   198 
   198 
       
   199 lemma greaterThanAtMost_empty[simp]:"l \<le> k ==> {k<..(l::'a::order)} = {}"
       
   200 by(auto simp:greaterThanAtMost_def greaterThan_def atMost_def)
       
   201 
       
   202 lemma greaterThanLessThan_empty[simp]:"l \<le> k ==> {k<..(l::'a::order)} = {}"
       
   203 by(auto simp:greaterThanLessThan_def greaterThan_def lessThan_def)
       
   204 
   199 lemma atLeastAtMost_singleton [simp]: "{a::'a::order..a} = {a}";
   205 lemma atLeastAtMost_singleton [simp]: "{a::'a::order..a} = {a}";
   200   by (auto simp add: atLeastAtMost_def atMost_def atLeast_def);
   206 by (auto simp add: atLeastAtMost_def atMost_def atLeast_def);
   201 
   207 
   202 subsection {* Intervals of natural numbers *}
   208 subsection {* Intervals of natural numbers *}
   203 
   209 
   204 subsubsection {* The Constant @{term lessThan} *}
   210 subsubsection {* The Constant @{term lessThan} *}
   205 
   211