Skip to content

Commit 1b80fd0

Browse files
committed
feat(Data/Quot): add surjective_quotient_mk (#12702)
add missing `surjective_quotient_mk` to mirror `surjective_quotient_mk'`, `Quotient.surjective_quotient_mk''`, and `surjective_quot_mk`.
1 parent 89472cc commit 1b80fd0

File tree

1 file changed

+5
-0
lines changed

1 file changed

+5
-0
lines changed

Mathlib/Data/Quot.lean

Lines changed: 5 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -347,6 +347,11 @@ theorem surjective_quot_mk (r : α → α → Prop) : Function.Surjective (Quot.
347347
Quot.exists_rep
348348
#align surjective_quot_mk surjective_quot_mk
349349

350+
/-- `Quotient.mk` is a surjective function. -/
351+
theorem surjective_quotient_mk {α : Sort*} (s : Setoid α) :
352+
Function.Surjective (Quotient.mk s) :=
353+
Quot.exists_rep
354+
350355
/-- `Quotient.mk'` is a surjective function. -/
351356
theorem surjective_quotient_mk' (α : Sort*) [s : Setoid α] :
352357
Function.Surjective (Quotient.mk' : α → Quotient s) :=

0 commit comments

Comments
 (0)