Zulip Chat Archive

Stream: Is there code for X?

Topic: zpow_succ


Kim Morrison (Mar 04 2024 at 04:41):

Where is

import Mathlib

theorem zpow_succ {G : Type} [Group G] (g : G) (x : Int) : g ^ (x + 1) = g * g ^ x := sorry

Kim Morrison (Mar 04 2024 at 04:41):

ugh, (mul_self_zpow g x).symm, okay

Kim Morrison (Mar 04 2024 at 04:42):

Seems weird to be missing this?

Jireh Loreaux (Mar 04 2024 at 04:56):

A little, but succ is slightly weird terminology to use for Int, right? I know we have docs#Int.succ, but I mean that we would normally use add_one.

Kim Morrison (Mar 04 2024 at 05:00):

Sure, zpow_add_one is fine.

Johan Commelin (Mar 04 2024 at 05:02):

I guess that lemma isn't very confluent with zpow_add? Should the RHS by g ^ x * g?

Yaël Dillies (Mar 04 2024 at 05:03):

Sorry, have you missed docs#zpow_add_one ?

Kim Morrison (Mar 04 2024 at 05:05):

Yes! :-)

Jireh Loreaux (Mar 04 2024 at 05:10):

Lol, I feel justified.


Last updated: May 02 2025 at 03:31 UTC