leanprover-community / mathlib

  • Home
  • Zulip archive
  • API documentation
  • Lean web editor
  • Links

Zulip Chat Archive

Stream: Is there code for X?

Topic: Fin counterpart of Nat.foldM


Jun Yoshida (Jul 22 2023 at 10:47):

Is there a Fin-counterpart of Nat.foldM?

universe u v
variable {α : Type u} {m : Type u → Type v} [Monad m]

example (n : Nat) (f : Fin n → α → m α) (init : α) : m α :=
  sorry

Last updated: May 02 2025 at 03:31 UTC

Theme Simple by wildflame © 2016 Powered by jekyll