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

Commit 850784c

Browse files
committed
chore(order/*): rename strict_mono_{incr,decr}_on to strict_{mono,anti}_on (#9401)
This was done as a direct find and replace
1 parent 1472799 commit 850784c

File tree

13 files changed

+102
-102
lines changed

13 files changed

+102
-102
lines changed

archive/100-theorems-list/73_ascending_descending_sequences.lean

Lines changed: 7 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -39,20 +39,20 @@ We then show the pair of labels must be unique. Now if there is no increasing se
3939
which is a contradiction if there are more than `r * s` elements.
4040
-/
4141
theorem erdos_szekeres {r s n : ℕ} {f : fin n → α} (hn : r * s < n) (hf : injective f) :
42-
(∃ (t : finset (fin n)), r < t.card ∧ strict_mono_incr_on f ↑t) ∨
43-
(∃ (t : finset (fin n)), s < t.card ∧ strict_mono_decr_on f ↑t) :=
42+
(∃ (t : finset (fin n)), r < t.card ∧ strict_mono_on f ↑t) ∨
43+
(∃ (t : finset (fin n)), s < t.card ∧ strict_anti_on f ↑t) :=
4444
begin
4545
-- Given an index `i`, produce the set of increasing (resp., decreasing) subsequences which ends
4646
-- at `i`.
4747
let inc_sequences_ending_in : fin n → finset (finset (fin n)) :=
48-
λ i, univ.powerset.filter (λ t, finset.max t = some i ∧ strict_mono_incr_on f ↑t),
48+
λ i, univ.powerset.filter (λ t, finset.max t = some i ∧ strict_mono_on f ↑t),
4949
let dec_sequences_ending_in : fin n → finset (finset (fin n)) :=
50-
λ i, univ.powerset.filter (λ t, finset.max t = some i ∧ strict_mono_decr_on f ↑t),
50+
λ i, univ.powerset.filter (λ t, finset.max t = some i ∧ strict_anti_on f ↑t),
5151
-- The singleton sequence is in both of the above collections.
5252
-- (This is useful to show that the maximum length subsequence is at least 1, and that the set
5353
-- of subsequences is nonempty.)
54-
have inc_i : ∀ i, {i} ∈ inc_sequences_ending_in i := λ i, by simp [strict_mono_incr_on],
55-
have dec_i : ∀ i, {i} ∈ dec_sequences_ending_in i := λ i, by simp [strict_mono_decr_on],
54+
have inc_i : ∀ i, {i} ∈ inc_sequences_ending_in i := λ i, by simp [strict_mono_on],
55+
have dec_i : ∀ i, {i} ∈ dec_sequences_ending_in i := λ i, by simp [strict_anti_on],
5656
-- Define the pair of labels: at index `i`, the pair is the maximum length of an increasing
5757
-- subsequence ending at `i`, paired with the maximum length of a decreasing subsequence ending
5858
-- at `i`.
@@ -110,7 +110,7 @@ begin
110110
apply le_of_lt ‹i < j› },
111111
-- To show it's increasing (i.e., `f` is monotone increasing on `t.insert j`), we do cases
112112
-- on what the possibilities could be - either in `t` or equals `j`.
113-
simp only [strict_mono_incr_on, strict_mono_decr_on, coe_insert, set.mem_insert_iff,
113+
simp only [strict_mono_on, strict_anti_on, coe_insert, set.mem_insert_iff,
114114
mem_coe],
115115
-- Most of the cases are just bashes.
116116
rintros x ⟨rfl | _⟩ y ⟨rfl | _⟩ _,

src/algebra/group_power/order.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -161,8 +161,8 @@ begin
161161
{ rw [←h, zero_pow Hnpos], apply pow_pos (by rwa ←h at Hxy : 0 < y),}
162162
end
163163

164-
theorem strict_mono_incr_on_pow {n : ℕ} (hn : 0 < n) :
165-
strict_mono_incr_on (λ x : R, x ^ n) (set.Ici 0) :=
164+
theorem strict_mono_on_pow {n : ℕ} (hn : 0 < n) :
165+
strict_mono_on (λ x : R, x ^ n) (set.Ici 0) :=
166166
λ x hx y hy h, pow_lt_pow_of_lt_left h hx hn
167167

168168
theorem one_le_pow_of_one_le {a : R} (H : 1 ≤ a) : ∀ (n : ℕ), 1 ≤ a ^ n
@@ -200,7 +200,7 @@ variable [linear_ordered_semiring R]
200200

201201
@[simp] theorem pow_left_inj {x y : R} {n : ℕ} (Hxpos : 0 ≤ x) (Hypos : 0 ≤ y) (Hnpos : 0 < n) :
202202
x ^ n = y ^ n ↔ x = y :=
203-
(@strict_mono_incr_on_pow R _ _ Hnpos).inj_on.eq_iff Hxpos Hypos
203+
(@strict_mono_on_pow R _ _ Hnpos).inj_on.eq_iff Hxpos Hypos
204204

205205
lemma lt_of_pow_lt_pow {a b : R} (n : ℕ) (hb : 0 ≤ b) (h : a ^ n < b ^ n) : a < b :=
206206
lt_of_not_ge $ λ hn, not_lt_of_ge (pow_le_pow_of_le_left hb hn _) h

src/algebra/order/field.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -695,7 +695,7 @@ lemma abs_inv (a : α) : abs a⁻¹ = (abs a)⁻¹ :=
695695
(abs_hom : monoid_with_zero_hom α α).map_inv' a
696696

697697
-- TODO: add lemmas with `a⁻¹`.
698-
lemma one_div_strict_mono_decr_on : strict_mono_decr_on (λ x : α, 1 / x) (set.Ioi 0) :=
698+
lemma one_div_strict_anti_on : strict_anti_on (λ x : α, 1 / x) (set.Ioi 0) :=
699699
λ x x1 y y1 xy, (one_div_lt_one_div (set.mem_Ioi.mp y1) (set.mem_Ioi.mp x1)).mpr xy
700700

701701
lemma one_div_pow_le_one_div_pow_of_le (a1 : 1 ≤ a) {m n : ℕ} (mn : m ≤ n) :

src/algebra/order/ring.lean

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -259,11 +259,11 @@ lemma mul_self_lt_mul_self (h1 : 0 ≤ a) (h2 : a < b) : a * a < b * b :=
259259
mul_lt_mul' h2.le h2 h1 $ h1.trans_lt h2
260260

261261
-- See Note [decidable namespace]
262-
protected lemma decidable.strict_mono_incr_on_mul_self [@decidable_rel α (≤)] :
263-
strict_mono_incr_on (λ x : α, x * x) (set.Ici 0) :=
262+
protected lemma decidable.strict_mono_on_mul_self [@decidable_rel α (≤)] :
263+
strict_mono_on (λ x : α, x * x) (set.Ici 0) :=
264264
λ x hx y hy hxy, decidable.mul_self_lt_mul_self hx hxy
265265

266-
lemma strict_mono_incr_on_mul_self : strict_mono_incr_on (λ x : α, x * x) (set.Ici 0) :=
266+
lemma strict_mono_on_mul_self : strict_mono_on (λ x : α, x * x) (set.Ici 0) :=
267267
λ x hx y hy hxy, mul_self_lt_mul_self hx hxy
268268

269269
-- See Note [decidable namespace]
@@ -1122,11 +1122,11 @@ by haveI := @linear_order.decidable_le α _; exact
11221122

11231123
lemma mul_self_lt_mul_self_iff {a b : α} (h1 : 0 ≤ a) (h2 : 0 ≤ b) : a < b ↔ a * a < b * b :=
11241124
by haveI := @linear_order.decidable_le α _; exact
1125-
((@decidable.strict_mono_incr_on_mul_self α _ _).lt_iff_lt h1 h2).symm
1125+
((@decidable.strict_mono_on_mul_self α _ _).lt_iff_lt h1 h2).symm
11261126

11271127
lemma mul_self_inj {a b : α} (h1 : 0 ≤ a) (h2 : 0 ≤ b) : a * a = b * b ↔ a = b :=
11281128
by haveI := @linear_order.decidable_le α _; exact
1129-
(@decidable.strict_mono_incr_on_mul_self α _ _).inj_on.eq_iff h1 h2
1129+
(@decidable.strict_mono_on_mul_self α _ _).inj_on.eq_iff h1 h2
11301130

11311131
@[simp] lemma mul_le_mul_left_of_neg {a b c : α} (h : c < 0) : c * a ≤ c * b ↔ b ≤ a :=
11321132
by haveI := @linear_order.decidable_le α _; exact

src/analysis/special_functions/exp_log.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -462,10 +462,10 @@ end
462462
lemma log_nonpos (hx : 0 ≤ x) (h'x : x ≤ 1) : log x ≤ 0 :=
463463
(log_nonpos_iff' hx).2 h'x
464464

465-
lemma strict_mono_incr_on_log : strict_mono_incr_on log (set.Ioi 0) :=
465+
lemma strict_mono_on_log : strict_mono_on log (set.Ioi 0) :=
466466
λ x hx y hy hxy, log_lt_log hx hxy
467467

468-
lemma strict_mono_decr_on_log : strict_mono_decr_on log (set.Iio 0) :=
468+
lemma strict_anti_on_log : strict_anti_on log (set.Iio 0) :=
469469
begin
470470
rintros x (hx : x < 0) y (hy : y < 0) hxy,
471471
rw [← log_abs y, ← log_abs x],
@@ -474,7 +474,7 @@ begin
474474
end
475475

476476
lemma log_inj_on_pos : set.inj_on log (set.Ioi 0) :=
477-
strict_mono_incr_on_log.inj_on
477+
strict_mono_on_log.inj_on
478478

479479
lemma eq_one_of_pos_of_log_eq_zero {x : ℝ} (h₁ : 0 < x) (h₂ : log x = 0) : x = 1 :=
480480
log_inj_on_pos (set.mem_Ioi.2 h₁) (set.mem_Ioi.2 zero_lt_one) (h₂.trans real.log_one.symm)

src/analysis/special_functions/trigonometric/arctan.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -120,7 +120,7 @@ univ_subset_iff.1 surj_on_tan
120120

121121
/-- `real.tan` as an `order_iso` between `(-(π / 2), π / 2)` and `ℝ`. -/
122122
def tan_order_iso : Ioo (-(π / 2)) (π / 2) ≃o ℝ :=
123-
(strict_mono_incr_on_tan.order_iso _ _).trans $ (order_iso.set_congr _ _ image_tan_Ioo).trans
123+
(strict_mono_on_tan.order_iso _ _).trans $ (order_iso.set_congr _ _ image_tan_Ioo).trans
124124
order_iso.set.univ
125125

126126
/-- Inverse of the `tan` function, returns values in the range `-π / 2 < arctan x` and

src/analysis/special_functions/trigonometric/basic.lean

Lines changed: 9 additions & 9 deletions
Original file line numberDiff line numberDiff line change
@@ -1281,29 +1281,29 @@ match (le_total x (π / 2) : x ≤ π / 2 ∨ π / 2 ≤ x), le_total y (π / 2)
12811281
apply cos_lt_cos_of_nonneg_of_le_pi_div_two; linarith)
12821282
end
12831283

1284-
lemma strict_mono_decr_on_cos : strict_mono_decr_on cos (Icc 0 π) :=
1284+
lemma strict_anti_on_cos : strict_anti_on cos (Icc 0 π) :=
12851285
λ x hx y hy hxy, cos_lt_cos_of_nonneg_of_le_pi hx.1 hy.2 hxy
12861286

12871287
lemma cos_le_cos_of_nonneg_of_le_pi {x y : ℝ} (hx₁ : 0 ≤ x) (hy₂ : y ≤ π) (hxy : x ≤ y) :
12881288
cos y ≤ cos x :=
1289-
(strict_mono_decr_on_cos.le_iff_le ⟨hx₁.trans hxy, hy₂⟩ ⟨hx₁, hxy.trans hy₂⟩).2 hxy
1289+
(strict_anti_on_cos.le_iff_le ⟨hx₁.trans hxy, hy₂⟩ ⟨hx₁, hxy.trans hy₂⟩).2 hxy
12901290

12911291
lemma sin_lt_sin_of_lt_of_le_pi_div_two {x y : ℝ} (hx₁ : -(π / 2) ≤ x)
12921292
(hy₂ : y ≤ π / 2) (hxy : x < y) : sin x < sin y :=
12931293
by rw [← cos_sub_pi_div_two, ← cos_sub_pi_div_two, ← cos_neg (x - _), ← cos_neg (y - _)];
12941294
apply cos_lt_cos_of_nonneg_of_le_pi; linarith
12951295

1296-
lemma strict_mono_incr_on_sin : strict_mono_incr_on sin (Icc (-(π / 2)) (π / 2)) :=
1296+
lemma strict_mono_on_sin : strict_mono_on sin (Icc (-(π / 2)) (π / 2)) :=
12971297
λ x hx y hy hxy, sin_lt_sin_of_lt_of_le_pi_div_two hx.1 hy.2 hxy
12981298

12991299
lemma sin_le_sin_of_le_of_le_pi_div_two {x y : ℝ} (hx₁ : -(π / 2) ≤ x)
13001300
(hy₂ : y ≤ π / 2) (hxy : x ≤ y) : sin x ≤ sin y :=
1301-
(strict_mono_incr_on_sin.le_iff_le ⟨hx₁, hxy.trans hy₂⟩ ⟨hx₁.trans hxy, hy₂⟩).2 hxy
1301+
(strict_mono_on_sin.le_iff_le ⟨hx₁, hxy.trans hy₂⟩ ⟨hx₁.trans hxy, hy₂⟩).2 hxy
13021302

13031303
lemma inj_on_sin : inj_on sin (Icc (-(π / 2)) (π / 2)) :=
1304-
strict_mono_incr_on_sin.inj_on
1304+
strict_mono_on_sin.inj_on
13051305

1306-
lemma inj_on_cos : inj_on cos (Icc 0 π) := strict_mono_decr_on_cos.inj_on
1306+
lemma inj_on_cos : inj_on cos (Icc 0 π) := strict_anti_on_cos.inj_on
13071307

13081308
lemma surj_on_sin : surj_on sin (Icc (-(π / 2)) (π / 2)) (Icc (-1) 1) :=
13091309
by simpa only [sin_neg, sin_pi_div_two]
@@ -1661,7 +1661,7 @@ end angle
16611661

16621662
/-- `real.sin` as an `order_iso` between `[-(π / 2), π / 2]` and `[-1, 1]`. -/
16631663
def sin_order_iso : Icc (-(π / 2)) (π / 2) ≃o Icc (-1:ℝ) 1 :=
1664-
(strict_mono_incr_on_sin.order_iso _ _).trans $ order_iso.set_congr _ _ bij_on_sin.image_eq
1664+
(strict_mono_on_sin.order_iso _ _).trans $ order_iso.set_congr _ _ bij_on_sin.image_eq
16651665

16661666
@[simp] lemma coe_sin_order_iso_apply (x : Icc (-(π / 2)) (π / 2)) :
16671667
(sin_order_iso x : ℝ) = sin x := rfl
@@ -1723,11 +1723,11 @@ match le_total x 0, le_total y 0 with
17231723
| or.inr hx0, or.inr hy0 := tan_lt_tan_of_nonneg_of_lt_pi_div_two hx0 hy₂ hxy
17241724
end
17251725

1726-
lemma strict_mono_incr_on_tan : strict_mono_incr_on tan (Ioo (-(π / 2)) (π / 2)) :=
1726+
lemma strict_mono_on_tan : strict_mono_on tan (Ioo (-(π / 2)) (π / 2)) :=
17271727
λ x hx y hy, tan_lt_tan_of_lt_of_lt_pi_div_two hx.1 hy.2
17281728

17291729
lemma inj_on_tan : inj_on tan (Ioo (-(π / 2)) (π / 2)) :=
1730-
strict_mono_incr_on_tan.inj_on
1730+
strict_mono_on_tan.inj_on
17311731

17321732
lemma tan_inj_of_lt_of_lt_pi_div_two {x y : ℝ} (hx₁ : -(π / 2) < x) (hx₂ : x < π / 2)
17331733
(hy₁ : -(π / 2) < y) (hy₂ : y < π / 2) (hxy : tan x = tan y) : x = y :=

src/analysis/special_functions/trigonometric/inverse.lean

Lines changed: 8 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -53,14 +53,14 @@ inj_on_sin (arcsin_mem_Icc _) hx $ by rw [sin_arcsin (neg_one_le_sin _) (sin_le_
5353
lemma arcsin_sin {x : ℝ} (hx₁ : -(π / 2) ≤ x) (hx₂ : x ≤ π / 2) : arcsin (sin x) = x :=
5454
arcsin_sin' ⟨hx₁, hx₂⟩
5555

56-
lemma strict_mono_incr_on_arcsin : strict_mono_incr_on arcsin (Icc (-1) 1) :=
57-
(subtype.strict_mono_coe _).comp_strict_mono_incr_on $
58-
sin_order_iso.symm.strict_mono.strict_mono_incr_on_Icc_extend _
56+
lemma strict_mono_on_arcsin : strict_mono_on arcsin (Icc (-1) 1) :=
57+
(subtype.strict_mono_coe _).comp_strict_mono_on $
58+
sin_order_iso.symm.strict_mono.strict_mono_on_Icc_extend _
5959

6060
lemma monotone_arcsin : monotone arcsin :=
6161
(subtype.mono_coe _).comp $ sin_order_iso.symm.monotone.Icc_extend _
6262

63-
lemma inj_on_arcsin : inj_on arcsin (Icc (-1) 1) := strict_mono_incr_on_arcsin.inj_on
63+
lemma inj_on_arcsin : inj_on arcsin (Icc (-1) 1) := strict_mono_on_arcsin.inj_on
6464

6565
lemma arcsin_inj {x y : ℝ} (hx₁ : -1 ≤ x) (hx₂ : x ≤ 1) (hy₁ : -1 ≤ y) (hy₂ : y ≤ 1) :
6666
arcsin x = arcsin y ↔ x = y :=
@@ -109,7 +109,7 @@ end
109109

110110
lemma arcsin_le_iff_le_sin {x y : ℝ} (hx : x ∈ Icc (-1 : ℝ) 1) (hy : y ∈ Icc (-(π / 2)) (π / 2)) :
111111
arcsin x ≤ y ↔ x ≤ sin y :=
112-
by rw [← arcsin_sin' hy, strict_mono_incr_on_arcsin.le_iff_le hx (sin_mem_Icc _), arcsin_sin' hy]
112+
by rw [← arcsin_sin' hy, strict_mono_on_arcsin.le_iff_le hx (sin_mem_Icc _), arcsin_sin' hy]
113113

114114
lemma arcsin_le_iff_le_sin' {x y : ℝ} (hy : y ∈ Ico (-(π / 2)) (π / 2)) :
115115
arcsin x ≤ y ↔ x ≤ sin y :=
@@ -355,10 +355,10 @@ by rw [arccos, cos_pi_div_two_sub, sin_arcsin hx₁ hx₂]
355355
lemma arccos_cos {x : ℝ} (hx₁ : 0 ≤ x) (hx₂ : x ≤ π) : arccos (cos x) = x :=
356356
by rw [arccos, ← sin_pi_div_two_sub, arcsin_sin]; simp [sub_eq_add_neg]; linarith
357357

358-
lemma strict_mono_decr_on_arccos : strict_mono_decr_on arccos (Icc (-1) 1) :=
359-
λ x hx y hy h, sub_lt_sub_left (strict_mono_incr_on_arcsin hx hy h) _
358+
lemma strict_anti_on_arccos : strict_anti_on arccos (Icc (-1) 1) :=
359+
λ x hx y hy h, sub_lt_sub_left (strict_mono_on_arcsin hx hy h) _
360360

361-
lemma arccos_inj_on : inj_on arccos (Icc (-1) 1) := strict_mono_decr_on_arccos.inj_on
361+
lemma arccos_inj_on : inj_on arccos (Icc (-1) 1) := strict_anti_on_arccos.inj_on
362362

363363
lemma arccos_inj {x y : ℝ} (hx₁ : -1 ≤ x) (hx₂ : x ≤ 1) (hy₁ : -1 ≤ y) (hy₂ : y ≤ 1) :
364364
arccos x = arccos y ↔ x = y :=

src/data/set/function.lean

Lines changed: 12 additions & 12 deletions
Original file line numberDiff line numberDiff line change
@@ -795,26 +795,26 @@ by simp
795795

796796
end set
797797

798-
lemma strict_mono_incr_on.inj_on [linear_order α] [preorder β] {f : α → β} {s : set α}
799-
(H : strict_mono_incr_on f s) :
798+
lemma strict_mono_on.inj_on [linear_order α] [preorder β] {f : α → β} {s : set α}
799+
(H : strict_mono_on f s) :
800800
s.inj_on f :=
801801
λ x hx y hy hxy, show ordering.eq.compares x y, from (H.compares hx hy).1 hxy
802802

803-
lemma strict_mono_decr_on.inj_on [linear_order α] [preorder β] {f : α → β} {s : set α}
804-
(H : strict_mono_decr_on f s) :
803+
lemma strict_anti_on.inj_on [linear_order α] [preorder β] {f : α → β} {s : set α}
804+
(H : strict_anti_on f s) :
805805
s.inj_on f :=
806-
@strict_mono_incr_on.inj_on α (order_dual β) _ _ f s H
806+
@strict_mono_on.inj_on α (order_dual β) _ _ f s H
807807

808-
lemma strict_mono_incr_on.comp [preorder α] [preorder β] [preorder γ]
809-
{g : β → γ} {f : α → β} {s : set α} {t : set β} (hg : strict_mono_incr_on g t)
810-
(hf : strict_mono_incr_on f s) (hs : set.maps_to f s t) :
811-
strict_mono_incr_on (g ∘ f) s :=
808+
lemma strict_mono_on.comp [preorder α] [preorder β] [preorder γ]
809+
{g : β → γ} {f : α → β} {s : set α} {t : set β} (hg : strict_mono_on g t)
810+
(hf : strict_mono_on f s) (hs : set.maps_to f s t) :
811+
strict_mono_on (g ∘ f) s :=
812812
λ x hx y hy hxy, hg (hs hx) (hs hy) $ hf hx hy hxy
813813

814-
lemma strict_mono.comp_strict_mono_incr_on [preorder α] [preorder β] [preorder γ]
814+
lemma strict_mono.comp_strict_mono_on [preorder α] [preorder β] [preorder γ]
815815
{g : β → γ} {f : α → β} {s : set α} (hg : strict_mono g)
816-
(hf : strict_mono_incr_on f s) :
817-
strict_mono_incr_on (g ∘ f) s :=
816+
(hf : strict_mono_on f s) :
817+
strict_mono_on (g ∘ f) s :=
818818
λ x hx y hy hxy, hg $ hf hx hy hxy
819819

820820
lemma strict_mono.cod_restrict [preorder α] [preorder β] {f : α → β} (hf : strict_mono f)

src/data/set/intervals/proj_Icc.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -60,7 +60,7 @@ 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) :=
63+
lemma strict_mono_on_proj_Icc : strict_mono_on (proj_Icc a b h) (Icc a b) :=
6464
λ x hx y hy hxy, by simpa only [proj_Icc_of_mem, hx, hy]
6565

6666
/-- Extend a function `[a, b] → β` to a map `α → β`. -/
@@ -104,6 +104,6 @@ variables [preorder β] {a b : α} (h : a ≤ b) {f : Icc a b → β}
104104
lemma monotone.Icc_extend (hf : monotone f) : monotone (Icc_extend h f) :=
105105
hf.comp $ monotone_proj_Icc h
106106

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)
107+
lemma strict_mono.strict_mono_on_Icc_extend (hf : strict_mono f) :
108+
strict_mono_on (Icc_extend h f) (Icc a b) :=
109+
hf.comp_strict_mono_on (strict_mono_on_proj_Icc h)

0 commit comments

Comments
 (0)