Skip to content

Commit

Permalink
Update src/Init/Control/Basic.lean
Browse files Browse the repository at this point in the history
  • Loading branch information
nomeata authored Apr 13, 2024
1 parent 82f7024 commit 8937dd5
Showing 1 changed file with 4 additions and 1 deletion.
5 changes: 4 additions & 1 deletion src/Init/Control/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -34,7 +34,10 @@ Error recovery and state can interact subtly. For example, the implementation of
-- NB: List instance is in mathlib. Once upstreamed, add
-- * `List`, where `failure` is the empty list and `<|>` concatenates.
class Alternative (f : Type u → Type v) extends Applicative f : Type (max (u+1) v) where
/-- See `Alternative`. -/
/--
Produces an empty collection or recoverable failure. The `<|>` operator collects values or recovers
from failures. See `Alternative` for more details.
-/
failure : {α : Type u} → f α
/--
Depending on the `Alternative` instance, collects values or recovers from `failure`s by
Expand Down

0 comments on commit 8937dd5

Please sign in to comment.