Skip to content

Commit

Permalink
Merge branch 'FR_setoid_instance' into FR_quotient_mk''_abbrev
Browse files Browse the repository at this point in the history
  • Loading branch information
FR-vdash-bot committed Sep 2, 2024
2 parents 94d8cdc + a92336b commit 8d146de
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Data/Quot.lean
Original file line number Diff line number Diff line change
Expand Up @@ -328,7 +328,7 @@ theorem surjective_quotient_mk {α : Sort*} (s : Setoid α) :
Quot.exists_rep

/-- `Quotient.mk'` is a surjective function. -/
theorem surjective_quotient_mk' (α : Sort*) {s : Setoid α} :
theorem surjective_quotient_mk' (α : Sort*) [s : Setoid α] :
Function.Surjective (Quotient.mk' : α → Quotient s) :=
Quot.exists_rep

Expand Down

0 comments on commit 8d146de

Please sign in to comment.