Skip to content

Commit

Permalink
chore(Data/Set/Image): [s : Setoid α] => {s : Setoid α} (#17588)
Browse files Browse the repository at this point in the history
  • Loading branch information
FR-vdash-bot committed Oct 9, 2024
1 parent ae74421 commit 17659b7
Showing 1 changed file with 1 addition and 2 deletions.
3 changes: 1 addition & 2 deletions Mathlib/Data/Set/Image.lean
Original file line number Diff line number Diff line change
Expand Up @@ -817,9 +817,8 @@ theorem range_quot_lift {r : ι → ι → Prop} (hf : ∀ x y, r x y → f x =
range (Quot.lift f hf) = range f :=
ext fun _ => (surjective_quot_mk _).exists

-- Porting note: the `Setoid α` instance is not being filled in
@[simp]
theorem range_quotient_mk [sa : Setoid α] : (range (α := Quotient sa) fun x : α => ⟦x⟧) = univ :=
theorem range_quotient_mk {s : Setoid α} : range (Quotient.mk s) = univ :=
range_quot_mk _

@[simp]
Expand Down

0 comments on commit 17659b7

Please sign in to comment.