Zulip Chat Archive
Stream: Is there code for X?
Topic: Pull predicate from has_mem expr
Ben (Oct 20 2022 at 20:15):
Part of a larger proof but what am I missing here:
example (A: Type) (G : Type*) [group G] (M: mul_action G A) (a: A) (g : G) : g ∈ stabilizer G a → (g • a = a) := begin
sorry
end
Yaël Dillies (Oct 20 2022 at 20:15):
docs#mul_action.mem_stabilizer_iff
Yaël Dillies (Oct 20 2022 at 20:16):
Or id
:stuck_out_tongue:
Last updated: Dec 20 2023 at 11:08 UTC