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

Commit 02b37b5

Browse files
committed
feat(group_theory/subgroup): eq_bot_of_card_eq (#8413)
Companion lemma to `eq_top_of_card_eq`.
1 parent 8a0d5e0 commit 02b37b5

File tree

1 file changed

+3
-0
lines changed

1 file changed

+3
-0
lines changed

src/group_theory/subgroup.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -422,6 +422,9 @@ begin
422422
congr
423423
end
424424

425+
@[to_additive] lemma eq_bot_of_card_eq [fintype H] (h : fintype.card H = 1) : H = ⊥ :=
426+
let _ := fintype.card_le_one_iff_subsingleton.mp (le_of_eq h) in by exactI eq_bot_of_subsingleton H
427+
425428
@[to_additive] lemma nontrivial_iff_exists_ne_one (H : subgroup G) :
426429
nontrivial H ↔ ∃ x ∈ H, x ≠ (1:G) :=
427430
subtype.nontrivial_iff_exists_ne (λ x, x ∈ H) (1 : H)

0 commit comments

Comments
 (0)