Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit e510b20

Browse files
committed
feat(group_theory/index): Index of intersection (#13186)
This PR adds `relindex_inf_le` and `index_inf_le`, which are companion lemmas to `relindex_inf_ne_zero` and `index_inf_ne_zero`.
1 parent cf131e1 commit e510b20

File tree

1 file changed

+12
-0
lines changed

1 file changed

+12
-0
lines changed

src/group_theory/index.lean

Lines changed: 12 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -232,6 +232,18 @@ begin
232232
exact relindex_inf_ne_zero hH hK,
233233
end
234234

235+
lemma relindex_inf_le : (H ⊓ K).relindex L ≤ H.relindex L * K.relindex L :=
236+
begin
237+
by_cases h : H.relindex L = 0,
238+
{ exact (le_of_eq (relindex_eq_zero_of_le_left (by exact inf_le_left) h)).trans (zero_le _) },
239+
rw [←inf_relindex_right, inf_assoc, ←relindex_mul_relindex _ _ L inf_le_right inf_le_right,
240+
inf_relindex_right, inf_relindex_right],
241+
exact mul_le_mul_right' (relindex_le_of_le_right inf_le_right h) (K.relindex L),
242+
end
243+
244+
lemma index_inf_le : (H ⊓ K).index ≤ H.index * K.index :=
245+
by simp_rw [←relindex_top_right, relindex_inf_le]
246+
235247
@[simp] lemma index_eq_one : H.index = 1 ↔ H = ⊤ :=
236248
⟨λ h, quotient_group.subgroup_eq_top_of_subsingleton H (cardinal.to_nat_eq_one_iff_unique.mp h).1,
237249
λ h, (congr_arg index h).trans index_top⟩

0 commit comments

Comments
 (0)