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

Commit 73b41b2

Browse files
urkudmergify[bot]
andauthored
chore(data/prod): rename injective_prod to injective.prod (#2058)
This way we can use dot notation Co-authored-by: mergify[bot] <37929162+mergify[bot]@users.noreply.github.com>
1 parent 6a6beaa commit 73b41b2

File tree

2 files changed

+2
-2
lines changed

2 files changed

+2
-2
lines changed

src/data/prod.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -87,6 +87,6 @@ end prod
8787

8888
open function
8989

90-
lemma function.injective_prod {f : α → γ} {g : β → δ} (hf : injective f) (hg : injective g) :
90+
lemma function.injective.prod {f : α → γ} {g : β → δ} (hf : injective f) (hg : injective g) :
9191
injective (λ p : α × β, (f p.1, g p.2)) :=
9292
assume ⟨a₁, b₁⟩ ⟨a₂, b₂⟩, by { simp [prod.mk.inj_iff],exact λ ⟨eq₁, eq₂⟩, ⟨hf eq₁, hg eq₂⟩ }

src/topology/uniform_space/uniform_embedding.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -157,7 +157,7 @@ lemma uniform_embedding_subtype_emb (p : α → Prop) {e : α → β} (ue : unif
157157
lemma uniform_embedding.prod {α' : Type*} {β' : Type*} [uniform_space α'] [uniform_space β']
158158
{e₁ : α → α'} {e₂ : β → β'} (h₁ : uniform_embedding e₁) (h₂ : uniform_embedding e₂) :
159159
uniform_embedding (λp:α×β, (e₁ p.1, e₂ p.2)) :=
160-
{ inj := function.injective_prod h₁.inj h₂.inj,
160+
{ inj := h₁.inj.prod h₂.inj,
161161
..h₁.to_uniform_inducing.prod h₂.to_uniform_inducing }
162162

163163
lemma is_complete_of_complete_image {m : α → β} {s : set α} (hm : uniform_inducing m)

0 commit comments

Comments
 (0)