Skip to content

Commit

Permalink
feat(group_theory/group_action/basic): Action on an orbit (#9220)
Browse files Browse the repository at this point in the history
A `mul_action` restricts to a `mul_action` on an orbit.
  • Loading branch information
tb65536 committed Sep 16, 2021
1 parent ca38357 commit 76f87b7
Showing 1 changed file with 10 additions and 0 deletions.
10 changes: 10 additions & 0 deletions src/group_theory/group_action/basic.lean
Expand Up @@ -133,6 +133,16 @@ variables {α} {β}
conv {to_rhs, rw [← hy, ← mul_one y, ← inv_mul_self x, ← mul_assoc,
mul_action.mul_smul, hx]}⟩⟩)⟩

@[to_additive] instance {b : β} : mul_action α (orbit α b) :=
{ smul := λ a b', ⟨a • b', orbit_eq_iff.mp (eq.trans (orbit_eq_iff.mpr (mem_orbit b' a))
(orbit_eq_iff.mpr b'.2))⟩,
one_smul := λ a, subtype.ext (one_smul α a),
mul_smul := λ a a' b', subtype.ext (mul_smul a a' b') }

@[simp, to_additive] lemma orbit.coe_smul {b : β} {a : α} {b' : orbit α b} :
↑(a • b') = a • (b' : β) :=
rfl

@[to_additive] lemma mem_fixed_points_iff_card_orbit_eq_one {a : β}
[fintype (orbit α a)] : a ∈ fixed_points α β ↔ fintype.card (orbit α a) = 1 :=
begin
Expand Down

0 comments on commit 76f87b7

Please sign in to comment.