Skip to content

Commit

Permalink
doc(group_theory/index): add a theorem name and fix a to_additive (#1…
Browse files Browse the repository at this point in the history
…0564)

I wanted to find the theorem I know as "Lagrange's theorem" but couldn't by searching.
This PR adds the name Lagrange's theorem to the relevant file, and also fixes an extra eager `to_additive` renaming that creates a lemma `add_subgroup.index_add_card` which talks about multiplication previously.
  • Loading branch information
alexjbest committed Dec 2, 2021
1 parent 7043521 commit 34758d3
Showing 1 changed file with 3 additions and 1 deletion.
4 changes: 3 additions & 1 deletion src/group_theory/index.lean
Expand Up @@ -11,6 +11,7 @@ import set_theory.fincard
# Index of a Subgroup
In this file we define the index of a subgroup, and prove several divisibility properties.
Several theorems proved in this file are known as Lagrange's theorem.
## Main definitions
Expand All @@ -21,6 +22,7 @@ In this file we define the index of a subgroup, and prove several divisibility p
# Main results
- `card_mul_index` : `nat.card H * H.index = nat.card G`
- `index_mul_card` : `H.index * fintype.card H = fintype.card G`
- `index_dvd_card` : `H.index ∣ fintype.card G`
- `index_eq_mul_of_le` : If `H ≤ K`, then `H.index = K.index * (H.subgroup_of K).index`
Expand Down Expand Up @@ -177,7 +179,7 @@ nat.dvd_antisymm (H.index_map_dvd hf1) (H.dvd_index_map hf2)
H.index = fintype.card (quotient_group.quotient H) :=
nat.card_eq_fintype_card

@[to_additive] lemma index_mul_card [fintype G] [hH : fintype H] :
@[to_additive index_mul_card] lemma index_mul_card [fintype G] [hH : fintype H] :
H.index * fintype.card H = fintype.card G :=
by rw [←relindex_bot_left_eq_card, ←index_bot_eq_card, mul_comm]; exact relindex_mul_index bot_le

Expand Down

0 comments on commit 34758d3

Please sign in to comment.