Skip to content

Commit 57ab210

Browse files
Update Cslib/Foundations/Data/FinFun.lean
Co-authored-by: Chris Henson <46805207+chenson2018@users.noreply.github.com>
1 parent bdc1e43 commit 57ab210

File tree

1 file changed

+2
-6
lines changed

1 file changed

+2
-6
lines changed

Cslib/Foundations/Data/FinFun.lean

Lines changed: 2 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -47,12 +47,8 @@ scoped notation:50 f "↾" support => FinFun.mkRestrictFun f support
4747
instance instFunLike [Zero β] : FunLike (α →₀ β) α β where
4848
coe f := f.fn
4949
coe_injective' := by
50-
rintro ⟨f1, support1, mem_support_fn1⟩ ⟨f2, support2, mem_support_fn2⟩
51-
simp only
52-
intro heq
53-
simp only [heq, mk.injEq, true_and]
54-
ext a
55-
grind
50+
rintro ⟨_, _⟩ ⟨_, _⟩
51+
simp_all [Finset.ext_iff]
5652

5753
@[scoped grind =]
5854
theorem coe_fn [Zero β] {f : α →₀ β} : (f : α → β) = f.fn := by simp [DFunLike.coe]

0 commit comments

Comments
 (0)