๐Ÿ“ฆ hediet / lean-experiments

๐Ÿ“„ Main.lean ยท 12 lines
1
2
3
4
5
6
7
8
9
10
11
12import Mathlib
import Lean
import CellularAutomatas.ca
import CellularAutomatas.common
import CellularAutomatas.defs
import CellularAutomatas.find_some

open Lean Elab Command Term Meta

def main : IO Unit :=
  IO.println "Hello, Lean World!"