src/HOL/Set_Interval.thy
changeset 50417 f18b92f91818
parent 47988 e4b69e10b990
child 50999 3de230ed0547
equal deleted inserted replaced
50413:bf01be7d1a44 50417:f18b92f91818
   348 lemma Int_greaterThanAtMost[simp]: "{a<..b} Int {c<..d} = {max a c <.. min b d}"
   348 lemma Int_greaterThanAtMost[simp]: "{a<..b} Int {c<..d} = {max a c <.. min b d}"
   349 by auto
   349 by auto
   350 
   350 
   351 lemma Int_greaterThanLessThan[simp]: "{a<..<b} Int {c<..<d} = {max a c <..< min b d}"
   351 lemma Int_greaterThanLessThan[simp]: "{a<..<b} Int {c<..<d} = {max a c <..< min b d}"
   352 by auto
   352 by auto
       
   353 
       
   354 lemma Int_atMost[simp]: "{..a} \<inter> {..b} = {.. min a b}"
       
   355   by (auto simp: min_def)
   353 
   356 
   354 end
   357 end
   355 
   358 
   356 
   359 
   357 subsection {* Intervals of natural numbers *}
   360 subsection {* Intervals of natural numbers *}