Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 80c7ac1

Browse files
committed
feat(algebra/big_operators/order): add fintype.sum_mono and fintype.sum_strict_mono (#6040)
1 parent a101788 commit 80c7ac1

File tree

1 file changed

+13
-0
lines changed

1 file changed

+13
-0
lines changed

src/algebra/big_operators/order.lean

Lines changed: 13 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -317,6 +317,19 @@ end canonically_ordered_comm_semiring
317317

318318
end finset
319319

320+
namespace fintype
321+
322+
variables [fintype α]
323+
324+
@[mono] lemma sum_mono [ordered_add_comm_monoid β] : monotone (λ f : α → β, ∑ x, f x) :=
325+
λ f g hfg, finset.sum_le_sum $ λ x _, hfg x
326+
327+
lemma sum_strict_mono [ordered_cancel_add_comm_monoid β] : strict_mono (λ f : α → β, ∑ x, f x) :=
328+
λ f g hfg, let ⟨hle, i, hlt⟩ := pi.lt_def.mp hfg in
329+
finset.sum_lt_sum (λ i _, hle i) ⟨i, finset.mem_univ i, hlt⟩
330+
331+
end fintype
332+
320333
namespace with_top
321334
open finset
322335

0 commit comments

Comments
 (0)