Skip to content

Commit

Permalink
feat(group_theory/subgroup/basic): add lemmas about subgroup.map (#…
Browse files Browse the repository at this point in the history
…17894)

Add lemmas about comparison of `map f H` and `map f K` that don't assume `injective f`.
  • Loading branch information
urkud committed Dec 13, 2022
1 parent a5c5166 commit 2be0e5f
Showing 1 changed file with 16 additions and 0 deletions.
16 changes: 16 additions & 0 deletions src/group_theory/subgroup/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2332,6 +2332,22 @@ lemma comap_map_eq_self_of_injective {f : G →* N} (h : function.injective f) (
comap f (map f H) = H :=
comap_map_eq_self (((ker_eq_bot_iff _).mpr h).symm ▸ bot_le)

@[to_additive]
lemma map_le_map_iff {f : G →* N} {H K : subgroup G} : H.map f ≤ K.map f ↔ H ≤ K ⊔ f.ker :=
by rw [map_le_iff_le_comap, comap_map_eq]

@[to_additive] lemma map_le_map_iff' {f : G →* N} {H K : subgroup G} :
H.map f ≤ K.map f ↔ H ⊔ f.ker ≤ K ⊔ f.ker :=
by simp only [map_le_map_iff, sup_le_iff, le_sup_right, and_true]

@[to_additive] lemma map_eq_map_iff {f : G →* N} {H K : subgroup G} :
H.map f = K.map f ↔ H ⊔ f.ker = K ⊔ f.ker :=
by simp only [le_antisymm_iff, map_le_map_iff']

@[to_additive] lemma map_eq_range_iff {f : G →* N} {H : subgroup G} :
H.map f = f.range ↔ codisjoint H f.ker :=
by rw [f.range_eq_map, map_eq_map_iff, codisjoint_iff, top_sup_eq]

@[to_additive]
lemma map_le_map_iff_of_injective {f : G →* N} (hf : function.injective f) {H K : subgroup G} :
H.map f ≤ K.map f ↔ H ≤ K :=
Expand Down

0 comments on commit 2be0e5f

Please sign in to comment.