Skip to content

Commit

Permalink
feat(group_theory/subgroup/basic): comap_le_comap lemmas (#14365)
Browse files Browse the repository at this point in the history
This PR adds some `comap_le_comap` lemmas.
  • Loading branch information
tb65536 committed May 31, 2022
1 parent 1b49d48 commit 111ce5b
Showing 1 changed file with 16 additions and 1 deletion.
17 changes: 16 additions & 1 deletion src/group_theory/subgroup/basic.lean
Expand Up @@ -2306,9 +2306,24 @@ lemma map_comap_eq_self_of_surjective {f : G →* N} (h : function.surjective f)
map f (comap f H) = H :=
map_comap_eq_self ((range_top_of_surjective _ h).symm ▸ le_top)

@[to_additive]
lemma comap_le_comap_of_le_range {f : G →* N} {K L : subgroup N} (hf : K ≤ f.range) :
K.comap f ≤ L.comap f ↔ K ≤ L :=
⟨(map_comap_eq_self hf).ge.trans ∘ map_le_iff_le_comap.mpr, comap_mono⟩

@[to_additive]
lemma comap_le_comap_of_surjective {f : G →* N} {K L : subgroup N} (hf : function.surjective f) :
K.comap f ≤ L.comap f ↔ K ≤ L :=
comap_le_comap_of_le_range (le_top.trans (f.range_top_of_surjective hf).ge)

@[to_additive]
lemma comap_lt_comap_of_surjective {f : G →* N} {K L : subgroup N} (hf : function.surjective f) :
K.comap f < L.comap f ↔ K < L :=
by simp_rw [lt_iff_le_not_le, comap_le_comap_of_surjective hf]

@[to_additive]
lemma comap_injective {f : G →* N} (h : function.surjective f) : function.injective (comap f) :=
λ K L hKL, by { apply_fun map f at hKL, simpa [map_comap_eq_self_of_surjective h] using hKL }
λ K L, by simp only [le_antisymm_iff, comap_le_comap_of_surjective h, imp_self]

@[to_additive]
lemma comap_map_eq_self {f : G →* N} {H : subgroup G} (h : f.ker ≤ H) :
Expand Down

0 comments on commit 111ce5b

Please sign in to comment.