Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Jul 28, 2024
1 parent 8d1b1ce commit c73ab6f
Show file tree
Hide file tree
Showing 2 changed files with 1 addition and 4 deletions.
2 changes: 1 addition & 1 deletion src/Init/Data/Subtype.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,7 +9,7 @@ import Init.Ext
namespace Subtype

universe u
variable {α : Type u} {p q : α → Prop}
variable {α : Sort u} {p q : α → Prop}

@[ext]
protected theorem ext : ∀ {a1 a2 : { x // p x }}, (a1 : α) = (a2 : α) → a1 = a2
Expand Down
3 changes: 0 additions & 3 deletions tests/lean/run/binop_binrel_perf_issue.lean
Original file line number Diff line number Diff line change
Expand Up @@ -58,9 +58,6 @@ section Mathlib.Data.Subtype

variable {α : Sort _} {p : α → Prop}

protected theorem Subtype.ext : ∀ {a1 a2 : { x // p x }}, (a1 : α) = (a2 : α) → a1 = a2
| ⟨_, _⟩, ⟨_, _⟩, rfl => rfl

theorem Subtype.coe_injective : Function.Injective (fun (a : Subtype p) ↦ (a : α)) := fun _ _ ↦ Subtype.ext

end Mathlib.Data.Subtype
Expand Down

0 comments on commit c73ab6f

Please sign in to comment.