Skip to content

Commit

Permalink
Merge pull request #21 from leanprover/bump_to_v4.14.0-rc1
Browse files Browse the repository at this point in the history
chore: adaptations for v4.14.0-rc1
  • Loading branch information
kim-em authored Nov 4, 2024
2 parents 2cf1030 + f905412 commit 726b3c9
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 5 deletions.
8 changes: 4 additions & 4 deletions Cli/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -256,7 +256,7 @@ section Configuration
parse? s := do
if s == ".lean" then
none
let name :=
let name :=
if s.endsWith ".lean" then
let pathComponents := (s : FilePath).withExtension "" |>.components
pathComponents.foldl .mkStr .anonymous
Expand Down Expand Up @@ -360,7 +360,7 @@ section Configuration
-/
structure Flag where
/-- Associated flag meta-data. -/
flag : Flag
flag : Cli.Flag
/-- Parsed value that was validated and conforms to `flag.type`. -/
value : String
deriving Inhabited, BEq, Repr
Expand Down Expand Up @@ -393,7 +393,7 @@ section Configuration
-/
structure Arg where
/-- Associated argument meta-data. -/
arg : Arg
arg : Cli.Arg
/-- Parsed value that was validated and conforms to `arg.type`. -/
value : String
deriving Inhabited, BEq, Repr
Expand Down Expand Up @@ -1630,4 +1630,4 @@ section IO
end Cmd
end IO

end Cli
end Cli
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:v4.9.0
leanprover/lean4:v4.14.0-rc1

0 comments on commit 726b3c9

Please sign in to comment.