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

Commit 155b315

Browse files
committed
chore(data/set/function): minor style fixes (#7027)
1 parent 44f34ee commit 155b315

File tree

1 file changed

+3
-3
lines changed

1 file changed

+3
-3
lines changed

src/data/set/function.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -260,7 +260,7 @@ lemma inj_on_iff_injective : inj_on f s ↔ injective (restrict f s) :=
260260
⟨λ H a b h, subtype.eq $ H a.2 b.2 h,
261261
λ H a as b bs h, congr_arg subtype.val $ @H ⟨a, as⟩ ⟨b, bs⟩ h⟩
262262

263-
lemma inj_on_preimage {B : set (set β)} (hB : B ⊆ powerset (range f)) :
263+
lemma inj_on_preimage {B : set (set β)} (hB : B ⊆ 𝒫 (range f)) :
264264
inj_on (preimage f) B :=
265265
λ s hs t ht hst, (preimage_eq_preimage' (hB hs) (hB ht)).1 hst
266266

@@ -436,7 +436,7 @@ theorem left_inv_on.inj_on (h : left_inv_on f₁' f s) : inj_on f s :=
436436
calc
437437
x₁ = f₁' (f x₁) : eq.symm $ h h₁
438438
... = f₁' (f x₂) : congr_arg f₁' heq
439-
... = x₂ : h h₂
439+
... = x₂ : h h₂
440440

441441
theorem left_inv_on.surj_on (h : left_inv_on f' f s) (hf : maps_to f s t) : surj_on f' t s :=
442442
λ x hx, ⟨f x, hf hx, h hx⟩
@@ -475,7 +475,7 @@ theorem left_inv_on.image_image (hf : left_inv_on f' f s) :
475475
f' '' (f '' s) = s :=
476476
by rw [image_image, image_congr hf, image_id']
477477

478-
theorem left_inv_on.image_image' (hf : left_inv_on f' f s) (hs : s₁ ⊆ s) :
478+
theorem left_inv_on.image_image' (hf : left_inv_on f' f s) (hs : s₁ ⊆ s) :
479479
f' '' (f '' s₁) = s₁ :=
480480
(hf.mono hs).image_image
481481

0 commit comments

Comments
 (0)