| changeset 66793 | deabce3ccf1f | 
| parent 65811 | 2653f1cd8775 | 
| child 66807 | c3631f32dfeb | 
--- a/src/HOL/Rings.thy Sun Oct 08 16:50:37 2017 +0200 +++ b/src/HOL/Rings.thy Mon Oct 09 15:34:23 2017 +0100 @@ -2241,6 +2241,10 @@ lemma minus_less_iff_1 [simp, no_atp]: "- a < 1 \<longleftrightarrow> - 1 < a" by (fact minus_less_iff) +lemma add_less_zeroD: + shows "x+y < 0 \<Longrightarrow> x<0 \<or> y<0" + by (auto simp: not_less intro: le_less_trans [of _ "x+y"]) + end text \<open>Simprules for comparisons where common factors can be cancelled.\<close>