src/HOL/Set_Interval.thy
changeset 56949 d1a937cbf858
parent 56480 093ea91498e6
child 57113 7e95523302e6
equal deleted inserted replaced
56948:1144d7ec892a 56949:d1a937cbf858
   464 by (auto simp: set_eq_iff intro: top_le)
   464 by (auto simp: set_eq_iff intro: top_le)
   465 
   465 
   466 lemma (in bounded_lattice) atLeastAtMost_eq_UNIV_iff:
   466 lemma (in bounded_lattice) atLeastAtMost_eq_UNIV_iff:
   467   "{x..y} = UNIV \<longleftrightarrow> (x = bot \<and> y = top)"
   467   "{x..y} = UNIV \<longleftrightarrow> (x = bot \<and> y = top)"
   468 by (auto simp: set_eq_iff intro: top_le le_bot)
   468 by (auto simp: set_eq_iff intro: top_le le_bot)
       
   469 
       
   470 lemma Iio_eq_empty_iff: "{..< n::'a::{linorder, order_bot}} = {} \<longleftrightarrow> n = bot"
       
   471   by (auto simp: set_eq_iff not_less le_bot)
       
   472 
       
   473 lemma Iio_eq_empty_iff_nat: "{..< n::nat} = {} \<longleftrightarrow> n = 0"
       
   474   by (simp add: Iio_eq_empty_iff bot_nat_def)
   469 
   475 
   470 
   476 
   471 subsection {* Infinite intervals *}
   477 subsection {* Infinite intervals *}
   472 
   478 
   473 context dense_linorder
   479 context dense_linorder