Skip to content

Commit

Permalink
feat(group_theory/subgroup/basic): disjoint_iff_mul_eq_one (#12505)
Browse files Browse the repository at this point in the history
  • Loading branch information
nomeata committed Mar 8, 2022
1 parent 1597e9a commit fac5ffe
Show file tree
Hide file tree
Showing 2 changed files with 30 additions and 0 deletions.
19 changes: 19 additions & 0 deletions src/group_theory/subgroup/basic.lean
Expand Up @@ -2731,6 +2731,25 @@ end

end subgroup_normal

@[to_additive]
lemma disjoint_def {H₁ H₂ : subgroup G} :
disjoint H₁ H₂ ↔ ∀ {x : G}, x ∈ H₁ → x ∈ H₂ → x = 1 :=
show (∀ x, x ∈ H₁ ∧ x ∈ H₂ → x ∈ ({1} : set G)) ↔ _, by simp

@[to_additive]
lemma disjoint_def' {H₁ H₂ : subgroup G} :
disjoint H₁ H₂ ↔ ∀ {x y : G}, x ∈ H₁ → y ∈ H₂ → x = y → x = 1 :=
disjoint_def.trans ⟨λ h x y hx hy hxy, h hx $ hxy.symm ▸ hy,
λ h x hx hx', h hx hx' rfl⟩

@[to_additive]
lemma disjoint_iff_mul_eq_one {H₁ H₂ : subgroup G} :
disjoint H₁ H₂ ↔ ∀ {x y : G}, x ∈ H₁ → y ∈ H₂ → x * y = 1 → x = 1 ∧ y = 1 :=
disjoint_def'.trans ⟨λ h x y hx hy hxy,
let hx1 : x = 1 := h hx (H₂.inv_mem hy) (eq_inv_iff_mul_eq_one.mpr hxy) in
⟨hx1, by simpa [hx1] using hxy⟩,
λ h x y hx hy hxy, (h hx (H₂.inv_mem hy) (mul_inv_eq_one.mpr hxy)).1

end subgroup

namespace is_conj
Expand Down
11 changes: 11 additions & 0 deletions src/group_theory/submonoid/basic.lean
Expand Up @@ -363,6 +363,17 @@ lemma supr_eq_closure {ι : Sort*} (p : ι → submonoid M) :
(⨆ i, p i) = submonoid.closure (⋃ i, (p i : set M)) :=
by simp_rw [submonoid.closure_Union, submonoid.closure_eq]

@[to_additive]
lemma disjoint_def {p₁ p₂ : submonoid M} :
disjoint p₁ p₂ ↔ ∀ {x : M}, x ∈ p₁ → x ∈ p₂ → x = 1 :=
show (∀ x, x ∈ p₁ ∧ x ∈ p₂ → x ∈ ({1} : set M)) ↔ _, by simp

@[to_additive]
lemma disjoint_def' {p₁ p₂ : submonoid M} :
disjoint p₁ p₂ ↔ ∀ {x y : M}, x ∈ p₁ → y ∈ p₂ → x = y → x = 1 :=
disjoint_def.trans ⟨λ h x y hx hy hxy, h hx $ hxy.symm ▸ hy,
λ h x hx hx', h hx hx' rfl⟩

end submonoid

namespace monoid_hom
Expand Down

0 comments on commit fac5ffe

Please sign in to comment.