Zulip Chat Archive
Stream: mathlib4
Topic: Another FunLike issue, with linear maps
Joël Riou (Apr 04 2023 at 09:34):
While trying to port Algebra.Category.Module.Basic
!4#3260, some basic instances are not found. Here is an example of the problem:
example {R M N : Type _} [Semiring R] [AddCommMonoid M] [Module R M]
[AddCommMonoid N] [Module R N] : FunLike (M →ₗ[R] N) M (fun _ => N) := inferInstance-- works
example {R M N : Type _} [Ring R] [AddCommGroup M] [Module R M]
[AddCommGroup N] [Module R N] : FunLike (M →ₗ[R] N) M (fun _ => N) := inferInstance --fails
Anne Baanen (Apr 04 2023 at 09:36):
Does (temporarily) enabling etaExperiment
help?
Matthew Ballard (Apr 04 2023 at 09:36):
Does attribute [-instance] Ring.toNonAssocRing in
fix it?
Joël Riou (Apr 04 2023 at 09:39):
Indeed, both etaExperiment
or -instance
work!
Moritz Doll (Apr 04 2023 at 09:39):
Can we have a 2074
emoji?
Last updated: Dec 20 2023 at 11:08 UTC