src/HOL/SupInf.thy
changeset 45966 03ce2b2a29a2
parent 44670 d1cb7bc44370
child 46757 ad878aff9c15
equal deleted inserted replaced
45965:2af982715e5c 45966:03ce2b2a29a2
   354 by auto (metis Inf_insert_nonempty z) 
   354 by auto (metis Inf_insert_nonempty z) 
   355 
   355 
   356 lemma Inf_greater:
   356 lemma Inf_greater:
   357   fixes z :: real
   357   fixes z :: real
   358   shows "X \<noteq> {} \<Longrightarrow> Inf X < z \<Longrightarrow> \<exists>x \<in> X. x < z"
   358   shows "X \<noteq> {} \<Longrightarrow> Inf X < z \<Longrightarrow> \<exists>x \<in> X. x < z"
   359   by (metis Inf_real_iff mem_def not_leE)
   359   by (metis Inf_real_iff not_leE)
   360 
   360 
   361 lemma Inf_close:
   361 lemma Inf_close:
   362   fixes e :: real
   362   fixes e :: real
   363   shows "X \<noteq> {} \<Longrightarrow> 0 < e \<Longrightarrow> \<exists>x \<in> X. x < Inf X + e"
   363   shows "X \<noteq> {} \<Longrightarrow> 0 < e \<Longrightarrow> \<exists>x \<in> X. x < Inf X + e"
   364   by (metis add_strict_increasing add_commute Inf_greater linorder_not_le pos_add_strict)
   364   by (metis add_strict_increasing add_commute Inf_greater linorder_not_le pos_add_strict)