Documentation

Mathlib.Data.Nat.Periodic

Periodic Functions on ℕ #

This file identifies a few functions on which are periodic, and also proves a lemma about periodic predicates which helps determine their cardinality when filtering intervals over them.

theorem Nat.periodic_mod (a : Nat) :
Function.Periodic (fun (n : Nat) => HMod.hMod n a) a
theorem Function.Periodic.map_mod_nat {α : Type u_1} {f : Natα} {a : Nat} (hf : Periodic f a) (n : Nat) :
Eq (f (HMod.hMod n a)) (f n)

An interval of length a filtered over a periodic predicate of period a has cardinality equal to the number naturals below a for which p a is true.

An interval of length a filtered over a periodic predicate of period a has cardinality equal to the number naturals below a for which p a is true.