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

Commit bf25d26

Browse files
committed
chore(data/set/intervals/proj_Icc): add strict_mono_incr_on (#5292)
* rename `set.Icc_extend_monotone` to `monotone.Icc_extend`; * add `set.strict_mono_incr_on_proj_Icc` and `strict_mono.strict_mono_incr_on_Icc_extend`.
1 parent efe18d5 commit bf25d26

File tree

1 file changed

+13
-3
lines changed

1 file changed

+13
-3
lines changed

src/data/set/intervals/proj_Icc.lean

Lines changed: 13 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -60,6 +60,9 @@ lemma proj_Icc_surjective : surjective (proj_Icc a b h) :=
6060
lemma monotone_proj_Icc : monotone (proj_Icc a b h) :=
6161
λ x y hxy, max_le_max le_rfl $ min_le_min le_rfl hxy
6262

63+
lemma strict_mono_incr_on_proj_Icc : strict_mono_incr_on (proj_Icc a b h) (Icc a b) :=
64+
λ x hx y hy hxy, by simpa only [proj_Icc_of_mem, hx, hy]
65+
6366
/-- Extend a function `[a, b] → β` to a map `α → β`. -/
6467
def Icc_extend {a b : α} (h : a ≤ b) (f : Icc a b → β) : α → β :=
6568
f ∘ proj_Icc a b h
@@ -92,8 +95,15 @@ congr_arg f $ proj_Icc_of_mem h hx
9295
Icc_extend h f x = f x :=
9396
congr_arg f $ proj_Icc_coe h x
9497

95-
lemma Icc_extend_monotone [preorder β] {f : Icc a b → β} (hf : monotone f) :
96-
monotone (Icc_extend h f) :=
98+
end set
99+
100+
open set
101+
102+
variables [preorder β] {a b : α} (h : a ≤ b) {f : Icc a b → β}
103+
104+
lemma monotone.Icc_extend (hf : monotone f) : monotone (Icc_extend h f) :=
97105
hf.comp $ monotone_proj_Icc h
98106

99-
end set
107+
lemma strict_mono.strict_mono_incr_on_Icc_extend (hf : strict_mono f) :
108+
strict_mono_incr_on (Icc_extend h f) (Icc a b) :=
109+
hf.comp_strict_mono_incr_on (strict_mono_incr_on_proj_Icc h)

0 commit comments

Comments
 (0)