Zulip Chat Archive

Stream: mathlib4

Topic: AlgEquiv.toFun_eq_coe


Antoine Chambert-Loir (Jul 29 2023 at 16:31):

Why did docs3#alg_equiv.to_fun_eq_coe disappear during the port from Mathlib3 to Mathlib4 ?

lemma AlgEquiv.toFun_eq_coe {R : Type u} {A₁ : Type v} {A₂ : Type w}
    [CommSemiring R] [Semiring A₁] [Semiring A₂]  [Algebra R A₁] [Algebra R A₂] (e : A₁ ≃ₐ[R] A₂)  :
  e.toFun = e := rfl

It's not that deep, but I found it useful in rewriting, and I did not find any swifter way than reintroducing it.

Kevin Buzzard (Jul 29 2023 at 16:38):

Probably because it became a syntactic equality in mathlib4 (or someone thought it did) so was no longer necessary? That's the usual reason coercion lemmas like this disappeared.

Antoine Chambert-Loir (Jul 29 2023 at 16:41):

Is there any objection to restoring it?
The point is that I need to apply map_one after that, but it is inaccessible otherwise.

Kevin Buzzard (Jul 29 2023 at 16:42):

Coercions work completely differently in mathlib4 to mathlib3. Are you sure that this is not a syntactic equality?

Kevin Buzzard (Jul 29 2023 at 16:45):

yeah the two sides are displaying differently, maybe this is an error and the lemma shouldn't have been deleted? The linter seems happy.

Notification Bot (Aug 07 2023 at 12:43):

17 messages were moved from this topic to #mathlib4 > Algebra.TensorProduct.rid as isomorphism over the larger ... by Eric Wieser.

Eric Wieser (Aug 07 2023 at 12:45):

Aside from the tangent I started (and now moved), we should definitely add back AlgEquiv.toFun_eq_coe


Last updated: Dec 20 2023 at 11:08 UTC