Skip to content

Commit

Permalink
fix: MLList.isEmpty's definition inversed (#1075)
Browse files Browse the repository at this point in the history
  • Loading branch information
crvdgc authored Dec 8, 2024
1 parent c016aa9 commit 74dffd1
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Batteries/Data/MLList/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -174,7 +174,7 @@ def fixl [Monad m] {α β : Type u} (f : α → m (α × List β)) (s : α) : ML

/-- Compute, inside the monad, whether a `MLList` is empty. -/
def isEmpty [Monad m] (xs : MLList m α) : m (ULift Bool) :=
(ULift.up ∘ Option.isSome) <$> uncons xs
(ULift.up ∘ Option.isNone) <$> uncons xs

/-- Convert a `List` to a `MLList`. -/
def ofList : List α → MLList m α
Expand Down

0 comments on commit 74dffd1

Please sign in to comment.