1339 end |
1339 end |
1340 |
1340 |
1341 |
1341 |
1342 subsection {* Tools setup *} |
1342 subsection {* Tools setup *} |
1343 |
1343 |
1344 lemma add_mono_thms_linordered_semiring [no_atp]: |
1344 lemma add_mono_thms_linordered_semiring: |
1345 fixes i j k :: "'a\<Colon>ordered_ab_semigroup_add" |
1345 fixes i j k :: "'a\<Colon>ordered_ab_semigroup_add" |
1346 shows "i \<le> j \<and> k \<le> l \<Longrightarrow> i + k \<le> j + l" |
1346 shows "i \<le> j \<and> k \<le> l \<Longrightarrow> i + k \<le> j + l" |
1347 and "i = j \<and> k \<le> l \<Longrightarrow> i + k \<le> j + l" |
1347 and "i = j \<and> k \<le> l \<Longrightarrow> i + k \<le> j + l" |
1348 and "i \<le> j \<and> k = l \<Longrightarrow> i + k \<le> j + l" |
1348 and "i \<le> j \<and> k = l \<Longrightarrow> i + k \<le> j + l" |
1349 and "i = j \<and> k = l \<Longrightarrow> i + k = j + l" |
1349 and "i = j \<and> k = l \<Longrightarrow> i + k = j + l" |
1350 by (rule add_mono, clarify+)+ |
1350 by (rule add_mono, clarify+)+ |
1351 |
1351 |
1352 lemma add_mono_thms_linordered_field [no_atp]: |
1352 lemma add_mono_thms_linordered_field: |
1353 fixes i j k :: "'a\<Colon>ordered_cancel_ab_semigroup_add" |
1353 fixes i j k :: "'a\<Colon>ordered_cancel_ab_semigroup_add" |
1354 shows "i < j \<and> k = l \<Longrightarrow> i + k < j + l" |
1354 shows "i < j \<and> k = l \<Longrightarrow> i + k < j + l" |
1355 and "i = j \<and> k < l \<Longrightarrow> i + k < j + l" |
1355 and "i = j \<and> k < l \<Longrightarrow> i + k < j + l" |
1356 and "i < j \<and> k \<le> l \<Longrightarrow> i + k < j + l" |
1356 and "i < j \<and> k \<le> l \<Longrightarrow> i + k < j + l" |
1357 and "i \<le> j \<and> k < l \<Longrightarrow> i + k < j + l" |
1357 and "i \<le> j \<and> k < l \<Longrightarrow> i + k < j + l" |