Zulip Chat Archive

Stream: new members

Topic: trivial kernel of injective monoid_hom


Yakov Pechersky (Jul 09 2021 at 23:53):

For a ->+ that is proven to be injective, what's the name of the lemma that the kernel is trivial? Specifically, I'm looking to prove this iff in a neat way

import group_theory.perm.basic

open equiv

variables {α β : Type*} {p : β  Prop} [decidable_pred p]

lemma extend_domain_eq_one_iff {e : perm α} {f : α  subtype p} :
  e.extend_domain f = 1  e = 1 :=
begin
end

Yakov Pechersky (Jul 09 2021 at 23:56):

Ah, monoid_hom.injective_iff.

Yakov Pechersky (Jul 10 2021 at 00:19):

Is there a reason why the RHS of the iff is in implication form instead of iff?

Eric Wieser (Jul 10 2021 at 04:53):

docs#monoid_hom.injective_iff

Eric Wieser (Jul 10 2021 at 04:54):

It's probably because if the RHS were an iff, then rw injective_iff leaves you a goal with more to clean up.


Last updated: Dec 20 2023 at 11:08 UTC