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.
1 parent 89472cc commit 1b80fd0Copy full SHA for 1b80fd0
Mathlib/Data/Quot.lean
@@ -347,6 +347,11 @@ theorem surjective_quot_mk (r : α → α → Prop) : Function.Surjective (Quot.
347
Quot.exists_rep
348
#align surjective_quot_mk surjective_quot_mk
349
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
+
355
/-- `Quotient.mk'` is a surjective function. -/
356
theorem surjective_quotient_mk' (α : Sort*) [s : Setoid α] :
357
Function.Surjective (Quotient.mk' : α → Quotient s) :=
0 commit comments