Skip to content

Commit 3128d20

Browse files
committed
feat: add @[grind inj] to Finset.coe_injective (#32714)
Requested at [#lean4 > `grind` doesn't use the fact that Prop is a Subsingleton @ 💬](https://leanprover.zulipchat.com/#narrow/channel/270676-lean4/topic/.60grind.60.20doesn't.20use.20the.20fact.20that.20Prop.20is.20a.20Subsingleton/near/555663373), seems reasonable.
1 parent 118bff1 commit 3128d20

File tree

1 file changed

+1
-0
lines changed

1 file changed

+1
-0
lines changed

Mathlib/Data/Finset/Defs.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -159,6 +159,7 @@ theorem ext {s₁ s₂ : Finset α} (h : ∀ a, a ∈ s₁ ↔ a ∈ s₂) : s
159159
theorem coe_inj {s₁ s₂ : Finset α} : (s₁ : Set α) = s₂ ↔ s₁ = s₂ :=
160160
SetLike.coe_set_eq
161161

162+
@[grind inj]
162163
theorem coe_injective {α} : Injective ((↑) : Finset α → Set α) := fun _s _t => coe_inj.1
163164

164165
/-! ### type coercion -/

0 commit comments

Comments
 (0)