Skip to content

Commit 916b76c

Browse files
committed
chore: address review comments
1 parent 360964b commit 916b76c

File tree

3 files changed

+8
-8
lines changed

3 files changed

+8
-8
lines changed

src/Lean/Shell.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1,13 +1,13 @@
11
/-
22
Copyright (c) 2025 Lean FRO. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
4-
Authors: eonardo de Moura, Mac Malone
4+
Authors: Leonardo de Moura, Mac Malone
55
-/
66
prelude
77
import Lean.Elab.Frontend
88
import Lean.Compiler.IR.EmitC
99

10-
/- Lean compaion to `shell.cpp` -/
10+
/- Lean companion to `shell.cpp` -/
1111

1212
open System
1313

@@ -26,7 +26,7 @@ private opaque initLLVM : IO Unit
2626

2727
/--
2828
Emits LLVM bitcode for the module.
29-
Before calling this function, the LLVM subsystem must first be successfuly initialized.
29+
Before calling this function, the LLVM subsystem must first be successfully initialized.
3030
-/
3131
@[extern "lean_emit_llvm"]
3232
private opaque emitLLVM (env : Environment) (modName : Name) (filepath : FilePath) : IO Unit

src/library/compiler/ir_interpreter.cpp

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1053,15 +1053,15 @@ class interpreter {
10531053
uint32 run_main(list_ref<string_ref> const & args) {
10541054
decl d = get_decl("main");
10551055
array_ref<param> const & params = decl_params(d);
1056-
buffer<object *> rargs;
1056+
buffer<object *> call_args;
10571057
if (params.size() == 2) { // List String -> IO _
1058-
rargs.push_back(args.to_obj_arg());
1058+
call_args.push_back(args.to_obj_arg());
10591059
} else { // IO _
10601060
lean_assert(params.size() == 1);
10611061
}
10621062
object * w = io_mk_world();
1063-
rargs.push_back(w);
1064-
w = call_boxed("main", rargs.size(), &rargs[0]);
1063+
call_args.push_back(w);
1064+
w = call_boxed("main", call_args.size(), &call_args[0]);
10651065
if (io_result_is_ok(w)) {
10661066
int ret = 0;
10671067
lean::expr ret_ty = m_env.get("main").get_type();

src/util/shell.cpp

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -356,7 +356,7 @@ uint32 run_shell_main(
356356
uint8_t json_output,
357357
array_ref<name> const & error_kinds,
358358
bool print_stats,
359-
optional<std::string> const & setup_file_name,
359+
optional<std::string> const & setup_file_name,
360360
bool run
361361
) {
362362
list_ref<string_ref> args;

0 commit comments

Comments
 (0)