diff --git a/.github/workflows/lean_action_ci.yml b/.github/workflows/lean_action_ci.yml new file mode 100644 index 0000000..09cd4ca --- /dev/null +++ b/.github/workflows/lean_action_ci.yml @@ -0,0 +1,14 @@ +name: Lean Action CI + +on: + push: + pull_request: + workflow_dispatch: + +jobs: + build: + runs-on: ubuntu-latest + + steps: + - uses: actions/checkout@v4 + - uses: leanprover/lean-action@v1 diff --git a/.gitignore b/.gitignore new file mode 100644 index 0000000..bfb30ec --- /dev/null +++ b/.gitignore @@ -0,0 +1 @@ +/.lake diff --git a/LeanSearchClient.lean b/LeanSearchClient.lean new file mode 100644 index 0000000..8464931 --- /dev/null +++ b/LeanSearchClient.lean @@ -0,0 +1,3 @@ +-- This module serves as the root of the `LeanSearchClient` library. +-- Import modules here that should be built as part of the library. +import LeanSearchClient.Basic \ No newline at end of file diff --git a/LeanSearchClient/Basic.lean b/LeanSearchClient/Basic.lean new file mode 100644 index 0000000..e99d3a6 --- /dev/null +++ b/LeanSearchClient/Basic.lean @@ -0,0 +1 @@ +def hello := "world" \ No newline at end of file diff --git a/Main.lean b/Main.lean new file mode 100644 index 0000000..4274768 --- /dev/null +++ b/Main.lean @@ -0,0 +1,4 @@ +import LeanSearchClient + +def main : IO Unit := + IO.println s!"Hello, {hello}!" diff --git a/README.md b/README.md new file mode 100644 index 0000000..6710b0d --- /dev/null +++ b/README.md @@ -0,0 +1 @@ +# LeanSearchClient \ No newline at end of file diff --git a/lakefile.lean b/lakefile.lean new file mode 100644 index 0000000..8a498d5 --- /dev/null +++ b/lakefile.lean @@ -0,0 +1,12 @@ +import Lake +open Lake DSL + +package "LeanSearchClient" where + -- add package configuration options here + +lean_lib «LeanSearchClient» where + -- add library configuration options here + +@[default_target] +lean_exe "leansearchclient" where + root := `Main diff --git a/lean-toolchain b/lean-toolchain new file mode 100644 index 0000000..5a9c76d --- /dev/null +++ b/lean-toolchain @@ -0,0 +1 @@ +leanprover/lean4:v4.11.0