Skip to content

Commit 410db90

Browse files
committed
fix(Logic/Embedding/Basic): Generalise arrowCongrRight_apply (#10739)
`f` does not need to be an embedding, and this version is syntactically strictly more general.
1 parent ea9e243 commit 410db90

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

Mathlib/Logic/Embedding/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -367,7 +367,7 @@ def arrowCongrRight {α : Sort u} {β : Sort v} {γ : Sort w} (e : α ↪ β) :
367367
#align function.embedding.arrow_congr_right Function.Embedding.arrowCongrRight
368368

369369
@[simp]
370-
theorem arrowCongrRight_apply {α : Sort u} {β : Sort v} {γ : Sort w} (e : α ↪ β) (f : γ α) :
370+
theorem arrowCongrRight_apply {α : Sort u} {β : Sort v} {γ : Sort w} (e : α ↪ β) (f : γ α) :
371371
arrowCongrRight e f = e ∘ f :=
372372
rfl
373373
#align function.embedding.arrow_congr_right_apply Function.Embedding.arrowCongrRight_apply

0 commit comments

Comments
 (0)