src/HOL/Real.thy
changeset 54262 326fd7103cb4
parent 54258 adfc759263ab
child 54263 c4159fe6fa46
equal deleted inserted replaced
54261:89991ef58448 54262:326fd7103cb4
   917     by (simp add: eq_Real `cauchy A` `cauchy B` width)
   917     by (simp add: eq_Real `cauchy A` `cauchy B` width)
   918   show "\<exists>y. (\<forall>x\<in>S. x \<le> y) \<and> (\<forall>z. (\<forall>x\<in>S. x \<le> z) \<longrightarrow> y \<le> z)"
   918   show "\<exists>y. (\<forall>x\<in>S. x \<le> y) \<and> (\<forall>z. (\<forall>x\<in>S. x \<le> z) \<longrightarrow> y \<le> z)"
   919     using 1 2 3 by (rule_tac x="Real B" in exI, simp)
   919     using 1 2 3 by (rule_tac x="Real B" in exI, simp)
   920 qed
   920 qed
   921 
   921 
   922 (* TODO: generalize to ordered group *)
       
   923 lemma bdd_above_uminus[simp]: "bdd_above (uminus ` X) \<longleftrightarrow> bdd_below (X::real set)"
       
   924   by (auto simp: bdd_above_def bdd_below_def intro: le_imp_neg_le) (metis le_imp_neg_le minus_minus)
       
   925 
       
   926 lemma bdd_below_uminus[simp]: "bdd_below (uminus ` X) \<longleftrightarrow> bdd_above (X::real set)"
       
   927   by (auto simp: bdd_above_def bdd_below_def intro: le_imp_neg_le) (metis le_imp_neg_le minus_minus)
       
   928 
       
   929 instantiation real :: linear_continuum
   922 instantiation real :: linear_continuum
   930 begin
   923 begin
   931 
   924 
   932 subsection{*Supremum of a set of reals*}
   925 subsection{*Supremum of a set of reals*}
   933 
   926