We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
arrowCongrRight_apply
1 parent ea9e243 commit 410db90Copy full SHA for 410db90
Mathlib/Logic/Embedding/Basic.lean
@@ -367,7 +367,7 @@ def arrowCongrRight {α : Sort u} {β : Sort v} {γ : Sort w} (e : α ↪ β) :
367
#align function.embedding.arrow_congr_right Function.Embedding.arrowCongrRight
368
369
@[simp]
370
-theorem arrowCongrRight_apply {α : Sort u} {β : Sort v} {γ : Sort w} (e : α ↪ β) (f : γ ↪ α) :
+theorem arrowCongrRight_apply {α : Sort u} {β : Sort v} {γ : Sort w} (e : α ↪ β) (f : γ → α) :
371
arrowCongrRight e f = e ∘ f :=
372
rfl
373
#align function.embedding.arrow_congr_right_apply Function.Embedding.arrowCongrRight_apply
0 commit comments