src/HOL/Real/RealDef.thy
changeset 25303 0699e20feabd
parent 25162 ad4d5365d9d8
child 25502 9200b36280c0
equal deleted inserted replaced
25302:19b1729f1bd4 25303:0699e20feabd
   415   show "x < y ==> 0 < z ==> z * x < z * y" by (rule real_mult_less_mono2)
   415   show "x < y ==> 0 < z ==> z * x < z * y" by (rule real_mult_less_mono2)
   416   show "\<bar>x\<bar> = (if x < 0 then -x else x)" by (simp only: real_abs_def)
   416   show "\<bar>x\<bar> = (if x < 0 then -x else x)" by (simp only: real_abs_def)
   417   show "sgn x = (if x=0 then 0 else if 0<x then 1 else - 1)"
   417   show "sgn x = (if x=0 then 0 else if 0<x then 1 else - 1)"
   418     by (simp only: real_sgn_def)
   418     by (simp only: real_sgn_def)
   419 qed
   419 qed
       
   420 
       
   421 instance real :: lordered_ab_group_add ..
   420 
   422 
   421 text{*The function @{term real_of_preal} requires many proofs, but it seems
   423 text{*The function @{term real_of_preal} requires many proofs, but it seems
   422 to be essential for proving completeness of the reals from that of the
   424 to be essential for proving completeness of the reals from that of the
   423 positive reals.*}
   425 positive reals.*}
   424 
   426