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

Commit f582298

Browse files
committed
feat(group_theory/subgroup/basic): zpowers_eq_bot (#14366)
This PR adds a lemma `zpowers_eq_bot`.
1 parent ebb5206 commit f582298

File tree

1 file changed

+4
-1
lines changed

1 file changed

+4
-1
lines changed

src/group_theory/subgroup/basic.lean

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -2667,10 +2667,13 @@ instance zpowers_is_commutative (g : G) : (zpowers g).is_commutative :=
26672667
⟨⟨λ ⟨_, _, h₁⟩ ⟨_, _, h₂⟩, by rw [subtype.ext_iff, coe_mul, coe_mul,
26682668
subtype.coe_mk, subtype.coe_mk, ←h₁, ←h₂, zpow_mul_comm]⟩⟩
26692669

2670-
@[simp, to_additive zmultiples_le, simp]
2670+
@[simp, to_additive zmultiples_le]
26712671
lemma zpowers_le {g : G} {H : subgroup G} : zpowers g ≤ H ↔ g ∈ H :=
26722672
by rw [zpowers_eq_closure, closure_le, set.singleton_subset_iff, set_like.mem_coe]
26732673

2674+
@[simp, to_additive zmultiples_eq_bot] lemma zpowers_eq_bot {g : G} : zpowers g = ⊥ ↔ g = 1 :=
2675+
by rw [eq_bot_iff, zpowers_le, mem_bot]
2676+
26742677
end subgroup
26752678

26762679
namespace monoid_hom

0 commit comments

Comments
 (0)