src/HOL/OrderedGroup.thy
changeset 29833 409138c4de12
parent 29670 cbe35f4f04f8
child 29886 b8a6b9c56fdd
equal deleted inserted replaced
29832:b4919260eaec 29833:409138c4de12
   596 
   596 
   597 lemma le_iff_diff_le_0: "a \<le> b \<longleftrightarrow> a - b \<le> 0"
   597 lemma le_iff_diff_le_0: "a \<le> b \<longleftrightarrow> a - b \<le> 0"
   598 by (simp add: algebra_simps)
   598 by (simp add: algebra_simps)
   599 
   599 
   600 text{*Legacy - use @{text algebra_simps} *}
   600 text{*Legacy - use @{text algebra_simps} *}
   601 lemmas group_simps = algebra_simps
   601 lemmas group_simps[noatp] = algebra_simps
   602 
   602 
   603 end
   603 end
   604 
   604 
   605 text{*Legacy - use @{text algebra_simps} *}
   605 text{*Legacy - use @{text algebra_simps} *}
   606 lemmas group_simps = algebra_simps
   606 lemmas group_simps[noatp] = algebra_simps
   607 
   607 
   608 class ordered_ab_semigroup_add =
   608 class ordered_ab_semigroup_add =
   609   linorder + pordered_ab_semigroup_add
   609   linorder + pordered_ab_semigroup_add
   610 
   610 
   611 class ordered_cancel_ab_semigroup_add =
   611 class ordered_cancel_ab_semigroup_add =
  1308     and "i < j \<and> k < l \<Longrightarrow> i + k < j + l"
  1308     and "i < j \<and> k < l \<Longrightarrow> i + k < j + l"
  1309 by (auto intro: add_strict_right_mono add_strict_left_mono
  1309 by (auto intro: add_strict_right_mono add_strict_left_mono
  1310   add_less_le_mono add_le_less_mono add_strict_mono)
  1310   add_less_le_mono add_le_less_mono add_strict_mono)
  1311 
  1311 
  1312 text{*Simplification of @{term "x-y < 0"}, etc.*}
  1312 text{*Simplification of @{term "x-y < 0"}, etc.*}
  1313 lemmas diff_less_0_iff_less [simp] = less_iff_diff_less_0 [symmetric]
  1313 lemmas diff_less_0_iff_less [simp, noatp] = less_iff_diff_less_0 [symmetric]
  1314 lemmas diff_eq_0_iff_eq [simp, noatp] = eq_iff_diff_eq_0 [symmetric]
  1314 lemmas diff_eq_0_iff_eq [simp, noatp] = eq_iff_diff_eq_0 [symmetric]
  1315 lemmas diff_le_0_iff_le [simp] = le_iff_diff_le_0 [symmetric]
  1315 lemmas diff_le_0_iff_le [simp, noatp] = le_iff_diff_le_0 [symmetric]
  1316 
  1316 
  1317 ML {*
  1317 ML {*
  1318 structure ab_group_add_cancel = Abel_Cancel
  1318 structure ab_group_add_cancel = Abel_Cancel
  1319 (
  1319 (
  1320 
  1320