Skip to content

Commit

Permalink
fix (LinearAlgebra.Dual): delete instFunLikeDual (#6637)
Browse files Browse the repository at this point in the history
It seems that Lean can find `LinearMap.instFunLike` just fine now. Furthermore, `Module.Dual.instFunLikeDual` was causing TC synthesis to fail. We delete it.
  • Loading branch information
mattrobball committed Aug 18, 2023
1 parent 05ef5b4 commit 971fb7a
Showing 1 changed file with 0 additions and 3 deletions.
3 changes: 0 additions & 3 deletions Mathlib/LinearAlgebra/Dual.lean
Expand Up @@ -124,9 +124,6 @@ namespace Dual

instance : Inhabited (Dual R M) := ⟨0

instance : FunLike (Dual R M) M fun _ => R :=
inferInstanceAs (FunLike (M →ₗ[R] R) M fun _ => R)

/-- Maps a module M to the dual of the dual of M. See `Module.erange_coe` and
`Module.evalEquiv`. -/
def eval : M →ₗ[R] Dual R (Dual R M) :=
Expand Down

0 comments on commit 971fb7a

Please sign in to comment.