Reservoir

leanprover/lean4-samples

Code samples for Lean 4

GitHub Link Documentation

Pick a version!

TODO: should show a time axes that allows the users to view, filter and click copy the lakefile config.

README

lean4-samples

Code samples for Lean 4.

Get started

In order to run these samples you need a working Lean 4 environment. See Quickstart instructions on how to set that up.

Hello world

Every language needs a simple hello world sample.

CSV Parser

CSV parser is the simplest practical CSV parser you can write in Lean.