Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

Commit

Permalink
Remove duplicate unique perm instance
Browse files Browse the repository at this point in the history
PR #8387 already gave this
  • Loading branch information
pechersky authored Jul 25, 2021
1 parent 36b5ca1 commit ac1353b
Showing 1 changed file with 0 additions and 3 deletions.
3 changes: 0 additions & 3 deletions src/data/equiv/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -179,9 +179,6 @@ equiv.equiv_subsingleton_cod
lemma perm.subsingleton_eq_refl [subsingleton α] (e : perm α) :
e = equiv.refl α := subsingleton.elim _ _

instance equiv.unique_of_subsingleton {α : Type*} [subsingleton α] : unique (α ≃ α) :=
unique_of_subsingleton (equiv.refl α)

/-- Transfer `decidable_eq` across an equivalence. -/
protected def decidable_eq (e : α ≃ β) [decidable_eq β] : decidable_eq α :=
e.injective.decidable_eq
Expand Down

0 comments on commit ac1353b

Please sign in to comment.