Skip to content

Commit

Permalink
Merge pull request #50 from semorrison/paths
Browse files Browse the repository at this point in the history
chore: correct some paths
  • Loading branch information
semorrison committed Aug 23, 2023
2 parents 7ba1dc3 + a65075e commit 685a4f1
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion init.sh
@@ -1,5 +1,5 @@
#!/bin/bash
git clone https://github.com/insightmind/LeanInk ./leanInk -q
git clone https://github.com/leanprover/LeanInk ./leanInk -q
cd leanInk
git fetch --tags -q
latestTag=$(git describe --tags `git rev-list --tags --max-count=1`)
Expand Down
2 changes: 1 addition & 1 deletion lakefile.lean
Expand Up @@ -55,7 +55,7 @@ def indexOf? [BEq α] (xs : List α) (s : α) (start := 0): Option Nat :=
| a :: tail => if a == s then some start else indexOf? tail s (start+1)

/-! Walk the `test` folder looking for every `.lean` file that's not a `lakefile` or part of an
`lean_package` and run `leanInk` on it. If `capture` is true then update the `.lean.leanInk.expected`
`lake-packages` and run `leanInk` on it. If `capture` is true then update the `.lean.leanInk.expected`
file, otherwise compare the new output to the expected output and return an error if they are
different. -/
def execute (leanInkExe: FilePath) (capture : Bool) : IO UInt32 := do
Expand Down

0 comments on commit 685a4f1

Please sign in to comment.