src/HOL/Hyperreal/HyperArith.thy
changeset 16924 04246269386e
parent 16417 9bc16273c2d4
child 17298 ad73fb6144cf
equal deleted inserted replaced
16923:2d9ebdc0c1ee 16924:04246269386e
    68 apply (subst hypreal_of_real_le_iff [symmetric])
    68 apply (subst hypreal_of_real_le_iff [symmetric])
    69 apply (simp (no_asm))
    69 apply (simp (no_asm))
    70 done
    70 done
    71 
    71 
    72 subsection{*Absolute Value Function for the Hyperreals*}
    72 subsection{*Absolute Value Function for the Hyperreals*}
    73 
       
    74 declare abs_mult [simp]
       
    75 
    73 
    76 lemma hrabs_add_less:
    74 lemma hrabs_add_less:
    77      "[| abs x < r; abs y < s |] ==> abs(x+y) < r + (s::hypreal)"
    75      "[| abs x < r; abs y < s |] ==> abs(x+y) < r + (s::hypreal)"
    78 by (simp add: abs_if split: split_if_asm)
    76 by (simp add: abs_if split: split_if_asm)
    79 
    77